src/Pure/Isar/isar_thy.ML
changeset 8236 df3f983f5858
parent 8227 d67db92897df
child 8349 611342539639
equal deleted inserted replaced
8235:a4fb9be6b19a 8236:df3f983f5858
   118   val begin_block: ProofHistory.T -> ProofHistory.T
   118   val begin_block: ProofHistory.T -> ProofHistory.T
   119   val next_block: ProofHistory.T -> ProofHistory.T
   119   val next_block: ProofHistory.T -> ProofHistory.T
   120   val end_block: ProofHistory.T -> ProofHistory.T
   120   val end_block: ProofHistory.T -> ProofHistory.T
   121   val defer: int option -> ProofHistory.T -> ProofHistory.T
   121   val defer: int option -> ProofHistory.T -> ProofHistory.T
   122   val prefer: int -> ProofHistory.T -> ProofHistory.T
   122   val prefer: int -> ProofHistory.T -> ProofHistory.T
   123   val tac: Method.text -> ProofHistory.T -> ProofHistory.T
   123   val apply: Method.text -> ProofHistory.T -> ProofHistory.T
   124   val then_tac: Method.text -> ProofHistory.T -> ProofHistory.T
   124   val apply_end: Method.text -> ProofHistory.T -> ProofHistory.T
   125   val proof: (Comment.interest * (Method.text * Comment.interest) option) * Comment.text
   125   val proof: (Comment.interest * (Method.text * Comment.interest) option) * Comment.text
   126     -> ProofHistory.T -> ProofHistory.T
   126     -> ProofHistory.T -> ProofHistory.T
   127   val qed: (Method.text * Comment.interest) option * Comment.text
   127   val qed: (Method.text * Comment.interest) option * Comment.text
   128     -> Toplevel.transition -> Toplevel.transition
   128     -> Toplevel.transition -> Toplevel.transition
   129   val terminal_proof: ((Method.text * Comment.interest) * (Method.text * Comment.interest) option)
   129   val terminal_proof: ((Method.text * Comment.interest) * (Method.text * Comment.interest) option)
   347 val end_block = ProofHistory.applys Proof.end_block;
   347 val end_block = ProofHistory.applys Proof.end_block;
   348 
   348 
   349 
   349 
   350 (* shuffle state *)
   350 (* shuffle state *)
   351 
   351 
   352 fun shuffle meth i = Method.refine_no_facts (Method.Basic (K (meth i))) o Proof.assert_no_chain;
   352 fun shuffle meth i = Method.refine (Method.Basic (K (meth i))) o Proof.assert_no_chain;
   353 
   353 
   354 fun defer i = ProofHistory.applys (shuffle Method.defer i);
   354 fun defer i = ProofHistory.applys (shuffle Method.defer i);
   355 fun prefer i = ProofHistory.applys (shuffle Method.prefer i);
   355 fun prefer i = ProofHistory.applys (shuffle Method.prefer i);
   356 
   356 
   357 
   357 
   358 (* backward steps *)
   358 (* backward steps *)
   359 
   359 
   360 fun tac m = ProofHistory.applys (Method.refine_no_facts m o Proof.assert_backward);
   360 fun apply m = ProofHistory.applys (Method.refine m o Proof.assert_backward);
   361 fun then_tac m = ProofHistory.applys (Method.refine m o Proof.assert_backward);
   361 fun apply_end m = ProofHistory.applys (Method.refine_end m o Proof.assert_forward);
   362 
   362 
   363 val proof = ProofHistory.applys o Method.proof o
   363 val proof = ProofHistory.applys o Method.proof o
   364   apsome Comment.ignore_interest o Comment.ignore_interest' o Comment.ignore;
   364   apsome Comment.ignore_interest o Comment.ignore_interest' o Comment.ignore;
   365 
   365 
   366 
   366