word_lib: re-sync with AFP; fix broken document

Also switched on document generation so we don't miss these in the future.

Signed-off-by: Gerwin Klein <gerwin.klein@data61.csiro.au>
This commit is contained in:
Gerwin Klein 2020-03-19 21:04:47 +08:00 committed by Gerwin Klein
parent adc22ae58f
commit 600836ec7f
3 changed files with 3 additions and 3 deletions

View File

@ -4,7 +4,7 @@
* SPDX-License-Identifier: BSD-2-Clause
*)
chapter "Distinct Proposition"
section "Distinct Proposition"
theory Distinct_Prop (* part of non-AFP Word_Lib *)
imports

View File

@ -7,7 +7,7 @@
chapter Lib
session Word_Lib (lib) = "HOL-Word" +
options [timeout = 150]
options [timeout = 150, document=pdf]
sessions
"HOL-Library"
"HOL-Eisbach"

View File

@ -1612,7 +1612,7 @@ lemma ucast_less_ucast:
apply simp
done
\<comment> \<open>This weaker version was previously called ucast_less_ucast. We retain it to
\<comment> \<open>This weaker version was previously called @{text ucast_less_ucast}. We retain it to
support existing proofs.\<close>
lemmas ucast_less_ucast_weak = ucast_less_ucast[OF order.strict_implies_order]