src/Doc/Prog_Prove/Logic.thy
changeset 63935 aa1fe1103ab8
parent 63414 beb987127d0f
child 67406 23307fd33906
equal deleted inserted replaced
63934:397b25cee74c 63935:aa1fe1103ab8
   338 \begin{itemize}
   338 \begin{itemize}
   339 \item By hand, using \indexed{@{text of}}{of}.
   339 \item By hand, using \indexed{@{text of}}{of}.
   340 The expression @{text"conjI[of \"a=b\" \"False\"]"}
   340 The expression @{text"conjI[of \"a=b\" \"False\"]"}
   341 instantiates the unknowns in @{thm[source] conjI} from left to right with the
   341 instantiates the unknowns in @{thm[source] conjI} from left to right with the
   342 two formulas @{text"a=b"} and @{text False}, yielding the rule
   342 two formulas @{text"a=b"} and @{text False}, yielding the rule
   343 @{thm[display,mode=Rule]conjI[of "a=b" False]}
   343 @{thm[display,mode=Rule,margin=100]conjI[of "a=b" False]}
   344 
   344 
   345 In general, @{text"th[of string\<^sub>1 \<dots> string\<^sub>n]"} instantiates
   345 In general, @{text"th[of string\<^sub>1 \<dots> string\<^sub>n]"} instantiates
   346 the unknowns in the theorem @{text th} from left to right with the terms
   346 the unknowns in the theorem @{text th} from left to right with the terms
   347 @{text string\<^sub>1} to @{text string\<^sub>n}.
   347 @{text string\<^sub>1} to @{text string\<^sub>n}.
   348 
   348