From 4f147cba894baa9e372e2b67211140b1a6f7b16c Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Fri, 19 Jun 2020 12:41:54 +0200 Subject: reorganize --- spartan/core/Spartan.thy | 31 +++++++++++++++++-------------- 1 file changed, 17 insertions(+), 14 deletions(-) (limited to 'spartan/core/Spartan.thy') diff --git a/spartan/core/Spartan.thy b/spartan/core/Spartan.thy index 55eb657..0a5fe4c 100644 --- a/spartan/core/Spartan.thy +++ b/spartan/core/Spartan.thy @@ -69,10 +69,13 @@ axiomatization app :: \o \ o \ o\ ("(1_ `_)" [120, 121] 120) syntax - "_Pi" :: \idt \ o \ o \ o\ ("(2\_: _./ _)" 30) - "_lam" :: \pttrns \ o \ o \ o\ ("(2\_: _./ _)" 30) - "_lam2" :: \pttrns \ o \ o \ o\ + "_Pi" :: \idts \ o \ o \ o\ ("(2\_: _./ _)" 30) + "_Pi2" :: \idts \ o \ o \ o\ + "_lam" :: \idts \ o \ o \ o\ ("(2\_: _./ _)" 30) + "_lam2" :: \idts \ o \ o \ o\ translations + "\x xs: A. B" \ "CONST Pi A (\x. _Pi2 xs A B)" + "_Pi2 x A B" \ "\x: A. B" "\x: A. B" \ "CONST Pi A (\x. B)" "\x xs: A. b" \ "CONST lam A (\x. _lam2 xs A b)" "_lam2 x A b" \ "\x: A. b" @@ -151,23 +154,23 @@ section \Proof commands\ named_theorems typechk -ML_file \lib/lib.ML\ -ML_file \lib/goals.ML\ -ML_file \lib/focus.ML\ -ML_file \lib/types.ML\ +ML_file \lib.ML\ +ML_file \goals.ML\ +ML_file \focus.ML\ +ML_file \types.ML\ section \Congruence automation\ consts "rhs" :: \'a\ ("..") -ML_file \lib/congruence.ML\ +ML_file \congruence.ML\ section \Methods\ -ML_file \lib/elimination.ML\ \ \elimination rules\ -ML_file \lib/cases.ML\ \ \case reasoning rules\ +ML_file \elimination.ML\ \ \elimination rules\ +ML_file \cases.ML\ \ \case reasoning rules\ named_theorems intros and comps lemmas @@ -177,7 +180,7 @@ lemmas [comps] = beta Sig_comp and [cong] = Pi_cong lam_cong Sig_cong -ML_file \lib/tactics.ML\ +ML_file \tactics.ML\ method_setup assumptions = \Scan.succeed (fn ctxt => SIMPLE_METHOD ( @@ -238,7 +241,7 @@ ML_file \~~/src/Tools/misc_legacy.ML\ ML_file \~~/src/Tools/IsaPlanner/isand.ML\ ML_file \~~/src/Tools/IsaPlanner/rw_inst.ML\ ML_file \~~/src/Tools/IsaPlanner/zipper.ML\ -ML_file \lib/eqsubst.ML\ +ML_file \eqsubst.ML\ \ \\rewrite\ method\ consts rewrite_HOLE :: "'a::{}" ("\") @@ -265,7 +268,7 @@ lemma imp_cong_eq: done ML_file \~~/src/HOL/Library/cconv.ML\ -ML_file \lib/rewrite.ML\ +ML_file \rewrite.ML\ \ \\reduce\ computes terms via judgmental equalities\ setup \map_theory_simpset (fn ctxt => ctxt addSolver (mk_solver "" typechk_tac))\ @@ -284,7 +287,7 @@ consts iarg :: \'a\ ("?") hole :: \'b\ ("{}") -ML_file \lib/implicits.ML\ +ML_file \implicits.ML\ attribute_setup implicit = \Scan.succeed Implicits.implicit_defs_attr\ -- cgit v1.2.3