src/Doc/Implementation/Isar.thy
changeset 59498 50b60f501b05
parent 58801 f420225a22d6
child 60754 02924903a6fd
equal deleted inserted replaced
59497:0c5cd369a643 59498:50b60f501b05
   364   fix A B :: bool
   364   fix A B :: bool
   365   assume a: A and b: B
   365   assume a: A and b: B
   366 
   366 
   367   have "A \<and> B"
   367   have "A \<and> B"
   368     apply (tactic \<open>rtac @{thm conjI} 1\<close>)
   368     apply (tactic \<open>rtac @{thm conjI} 1\<close>)
   369     using a apply (tactic \<open>resolve_tac facts 1\<close>)
   369     using a apply (tactic \<open>resolve_tac @{context} facts 1\<close>)
   370     using b apply (tactic \<open>resolve_tac facts 1\<close>)
   370     using b apply (tactic \<open>resolve_tac @{context} facts 1\<close>)
   371     done
   371     done
   372 
   372 
   373   have "A \<and> B"
   373   have "A \<and> B"
   374     using a and b
   374     using a and b
   375     ML_val \<open>@{Isar.goal}\<close>
   375     ML_val \<open>@{Isar.goal}\<close>