src/HOL/Modelcheck/MuckeSyn.thy
changeset 26939 1035c89b4c02
parent 26342 0f65fa163304
child 26957 e3f04fdd994d
equal deleted inserted replaced
26938:64e850c3da9e 26939:1035c89b4c02
   195 (* extension with removing bold font (TH) *)
   195 (* extension with removing bold font (TH) *)
   196 fun mk_lam_def (_::_) _ _ = NONE  
   196 fun mk_lam_def (_::_) _ _ = NONE  
   197   | mk_lam_def [] ((Const("==",_) $ (Const _)) $ RHS) t = SOME t
   197   | mk_lam_def [] ((Const("==",_) $ (Const _)) $ RHS) t = SOME t
   198   | mk_lam_def [] ((Const("==",_) $ LHS) $ RHS) t = 
   198   | mk_lam_def [] ((Const("==",_) $ LHS) $ RHS) t = 
   199     let val thy = theory_of_thm t;
   199     let val thy = theory_of_thm t;
   200 	val fnam = Sign.string_of_term thy (getfun LHS);
   200 	val fnam = Syntax.string_of_term_global thy (getfun LHS);
   201 	val rhs = Sign.string_of_term thy (freeze_thaw RHS)
   201 	val rhs = Syntax.string_of_term_global thy (freeze_thaw RHS)
   202 	val gl = delete_bold_string (fnam ^" == % " ^ (getargs LHS) ^" . " ^ rhs);
   202 	val gl = delete_bold_string (fnam ^" == % " ^ (getargs LHS) ^" . " ^ rhs);
   203     in
   203     in
   204 	SOME (prove_goal thy gl (fn prems =>
   204 	SOME (prove_goal thy gl (fn prems =>
   205   		[(REPEAT (rtac ext_rl 1)), (rtac t 1) ]))
   205   		[(REPEAT (rtac ext_rl 1)), (rtac t 1) ]))
   206     end
   206     end