mirror of
https://github.com/swc-project/swc.git
synced 2024-12-29 00:23:10 +03:00
fix(es/minifier): Consider more aliases in sequences pass (#4583)
This commit is contained in:
parent
ad6b71150e
commit
3521ce09e7
@ -1,5 +1,5 @@
|
||||
class X {
|
||||
}
|
||||
function foo(t, t2) {}
|
||||
var c1 = new X();
|
||||
foo(c1, new X()), foo(c1, c1);
|
||||
var c1 = new X(), d1 = new X();
|
||||
foo(c1, d1), foo(c1, c1);
|
||||
|
@ -10,5 +10,5 @@ var C = function() {
|
||||
swcHelpers.classCallCheck(this, X);
|
||||
};
|
||||
function foo(t, t2) {}
|
||||
var c1 = new X();
|
||||
foo(c1, new X()), foo(c1, c1);
|
||||
var c1 = new X(), d1 = new X();
|
||||
foo(c1, d1), foo(c1, c1);
|
||||
|
@ -117,9 +117,9 @@ var ItemsList = function(_Component) {
|
||||
if (!swcHelpers._instanceof(instance, Constructor)) throw new TypeError("Cannot call a class as a function");
|
||||
}(this, ItemsList1);
|
||||
for(var _len = arguments.length, args = new Array(_len), _key = 0; _key < _len; _key++)args[_key] = arguments[_key];
|
||||
return _defineProperty(_assertThisInitialized(_this = _super.call.apply(_super, [
|
||||
return _this = _super.call.apply(_super, [
|
||||
this
|
||||
].concat(args))), "storeHighlightedItemReference", function(highlightedItem) {
|
||||
].concat(args)), _defineProperty(_assertThisInitialized(_this), "storeHighlightedItemReference", function(highlightedItem) {
|
||||
_this.props.onHighlightedItemChange(null === highlightedItem ? null : highlightedItem.item);
|
||||
}), _this;
|
||||
}
|
||||
|
@ -4,6 +4,6 @@ import { useRouter as d } from "next/router";
|
||||
import { useProject as e } from "@swr/use-project";
|
||||
import f from "@swr/use-team";
|
||||
export default function g() {
|
||||
var c = e(d().query.project).data;
|
||||
var g = d().query.project, c = e(g).data;
|
||||
return f().teamSlug, useProjectBranches(null == c ? void 0 : c.id).data, a(b, {});
|
||||
};
|
||||
|
45
crates/swc_ecma_minifier/src/alias/ctx.rs
Normal file
45
crates/swc_ecma_minifier/src/alias/ctx.rs
Normal file
@ -0,0 +1,45 @@
|
||||
use std::ops::{Deref, DerefMut};
|
||||
|
||||
use super::InfectionCollector;
|
||||
|
||||
impl<'a> InfectionCollector<'a> {
|
||||
pub(super) fn with_ctx(&mut self, ctx: Ctx) -> WithCtx<'_, 'a> {
|
||||
let orig_ctx = self.ctx;
|
||||
self.ctx = ctx;
|
||||
|
||||
WithCtx {
|
||||
analyzer: self,
|
||||
orig_ctx,
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
#[derive(Debug, Default, Clone, Copy)]
|
||||
pub(super) struct Ctx {
|
||||
pub track_expr_ident: bool,
|
||||
}
|
||||
|
||||
pub(super) struct WithCtx<'a, 'b> {
|
||||
analyzer: &'a mut InfectionCollector<'b>,
|
||||
orig_ctx: Ctx,
|
||||
}
|
||||
|
||||
impl<'a, 'b> Deref for WithCtx<'a, 'b> {
|
||||
type Target = InfectionCollector<'b>;
|
||||
|
||||
fn deref(&self) -> &Self::Target {
|
||||
self.analyzer
|
||||
}
|
||||
}
|
||||
|
||||
impl<'a, 'b> DerefMut for WithCtx<'a, 'b> {
|
||||
fn deref_mut(&mut self) -> &mut Self::Target {
|
||||
self.analyzer
|
||||
}
|
||||
}
|
||||
|
||||
impl Drop for WithCtx<'_, '_> {
|
||||
fn drop(&mut self) {
|
||||
self.analyzer.ctx = self.orig_ctx;
|
||||
}
|
||||
}
|
218
crates/swc_ecma_minifier/src/alias/mod.rs
Normal file
218
crates/swc_ecma_minifier/src/alias/mod.rs
Normal file
@ -0,0 +1,218 @@
|
||||
#![allow(clippy::needless_update)]
|
||||
|
||||
use rustc_hash::FxHashSet;
|
||||
use swc_atoms::js_word;
|
||||
use swc_common::{collections::AHashSet, SyntaxContext};
|
||||
use swc_ecma_ast::*;
|
||||
use swc_ecma_utils::{collect_decls, ident::IdentLike, BindingCollector};
|
||||
use swc_ecma_visit::{noop_visit_type, Visit, VisitWith};
|
||||
|
||||
use self::ctx::Ctx;
|
||||
use crate::marks::Marks;
|
||||
|
||||
mod ctx;
|
||||
|
||||
pub(crate) struct AliasConfig {
|
||||
#[allow(unused)]
|
||||
pub marks: Marks,
|
||||
}
|
||||
|
||||
pub(crate) fn collect_infects_from<N>(node: &N, config: AliasConfig) -> FxHashSet<Id>
|
||||
where
|
||||
N: for<'aa> VisitWith<InfectionCollector<'aa>>,
|
||||
N: VisitWith<BindingCollector<Id>>,
|
||||
{
|
||||
let unresolved_ctxt = SyntaxContext::empty().apply_mark(config.marks.unresolved_mark);
|
||||
let decls = collect_decls(node);
|
||||
|
||||
let mut visitor = InfectionCollector {
|
||||
config,
|
||||
unresolved_ctxt,
|
||||
|
||||
exclude: &decls,
|
||||
ctx: Default::default(),
|
||||
aliases: FxHashSet::default(),
|
||||
};
|
||||
|
||||
node.visit_with(&mut visitor);
|
||||
|
||||
visitor.aliases
|
||||
}
|
||||
|
||||
pub(crate) struct InfectionCollector<'a> {
|
||||
#[allow(unused)]
|
||||
config: AliasConfig,
|
||||
unresolved_ctxt: SyntaxContext,
|
||||
|
||||
exclude: &'a AHashSet<Id>,
|
||||
|
||||
ctx: Ctx,
|
||||
|
||||
aliases: FxHashSet<Id>,
|
||||
}
|
||||
|
||||
impl InfectionCollector<'_> {
|
||||
fn add_id(&mut self, e: &Id) {
|
||||
if self.exclude.contains(e) {
|
||||
return;
|
||||
}
|
||||
|
||||
if self.unresolved_ctxt == e.1 {
|
||||
match e.0 {
|
||||
js_word!("String")
|
||||
| js_word!("Object")
|
||||
| js_word!("Number")
|
||||
| js_word!("BigInt")
|
||||
| js_word!("Boolean")
|
||||
| js_word!("Math")
|
||||
| js_word!("Error") => return,
|
||||
_ => {}
|
||||
}
|
||||
}
|
||||
|
||||
self.aliases.insert(e.clone());
|
||||
}
|
||||
}
|
||||
|
||||
impl Visit for InfectionCollector<'_> {
|
||||
noop_visit_type!();
|
||||
|
||||
fn visit_bin_expr(&mut self, e: &BinExpr) {
|
||||
match e.op {
|
||||
op!("in")
|
||||
| op!("instanceof")
|
||||
| op!(bin, "-")
|
||||
| op!(bin, "+")
|
||||
| op!("/")
|
||||
| op!("*")
|
||||
| op!("%")
|
||||
| op!("&")
|
||||
| op!("^")
|
||||
| op!("|")
|
||||
| op!("==")
|
||||
| op!("===")
|
||||
| op!("!=")
|
||||
| op!("!==")
|
||||
| op!("<")
|
||||
| op!("<=")
|
||||
| op!(">")
|
||||
| op!(">=")
|
||||
| op!("<<")
|
||||
| op!(">>")
|
||||
| op!(">>>") => {
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: false,
|
||||
..self.ctx
|
||||
};
|
||||
e.visit_children_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
_ => {
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: true,
|
||||
..self.ctx
|
||||
};
|
||||
e.visit_children_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
fn visit_cond_expr(&mut self, e: &CondExpr) {
|
||||
{
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: false,
|
||||
..self.ctx
|
||||
};
|
||||
e.test.visit_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
|
||||
{
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: true,
|
||||
..self.ctx
|
||||
};
|
||||
e.cons.visit_with(&mut *self.with_ctx(ctx));
|
||||
e.alt.visit_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
}
|
||||
|
||||
fn visit_expr(&mut self, e: &Expr) {
|
||||
match e {
|
||||
Expr::Ident(i) => {
|
||||
if self.ctx.track_expr_ident {
|
||||
self.add_id(&i.to_id());
|
||||
}
|
||||
}
|
||||
|
||||
_ => {
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: true,
|
||||
..self.ctx
|
||||
};
|
||||
e.visit_children_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
fn visit_member_expr(&mut self, n: &MemberExpr) {
|
||||
{
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: false,
|
||||
..self.ctx
|
||||
};
|
||||
n.obj.visit_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
|
||||
{
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: false,
|
||||
..self.ctx
|
||||
};
|
||||
n.prop.visit_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
}
|
||||
|
||||
fn visit_member_prop(&mut self, n: &MemberProp) {
|
||||
if let MemberProp::Computed(c) = &n {
|
||||
c.visit_with(self);
|
||||
}
|
||||
}
|
||||
|
||||
fn visit_super_prop_expr(&mut self, n: &SuperPropExpr) {
|
||||
if let SuperProp::Computed(c) = &n.prop {
|
||||
c.visit_with(self);
|
||||
}
|
||||
}
|
||||
|
||||
fn visit_unary_expr(&mut self, e: &UnaryExpr) {
|
||||
match e.op {
|
||||
op!("~")
|
||||
| op!(unary, "-")
|
||||
| op!(unary, "+")
|
||||
| op!("!")
|
||||
| op!("typeof")
|
||||
| op!("void") => {
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: false,
|
||||
..self.ctx
|
||||
};
|
||||
e.visit_children_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
|
||||
_ => {
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: true,
|
||||
..self.ctx
|
||||
};
|
||||
e.visit_children_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
fn visit_update_expr(&mut self, e: &UpdateExpr) {
|
||||
let ctx = Ctx {
|
||||
track_expr_ident: false,
|
||||
..self.ctx
|
||||
};
|
||||
e.arg.visit_with(&mut *self.with_ctx(ctx));
|
||||
}
|
||||
}
|
@ -1,10 +1,11 @@
|
||||
use rustc_hash::FxHashSet;
|
||||
use swc_atoms::{js_word, JsWord};
|
||||
use swc_common::{
|
||||
collections::{AHashMap, AHashSet},
|
||||
SyntaxContext,
|
||||
};
|
||||
use swc_ecma_ast::*;
|
||||
use swc_ecma_utils::{collect_decls, find_ids, ident::IdentLike, Id, IsEmpty};
|
||||
use swc_ecma_utils::{collect_decls, find_ids, ident::IdentLike, BindingCollector, Id, IsEmpty};
|
||||
use swc_ecma_visit::{noop_visit_type, Visit, VisitWith};
|
||||
use swc_timer::timer;
|
||||
|
||||
@ -14,7 +15,7 @@ use self::{
|
||||
};
|
||||
use crate::{
|
||||
marks::Marks,
|
||||
util::{can_end_conditionally, idents_used_by},
|
||||
util::{can_end_conditionally, idents_used_by, IdentUsageCollector},
|
||||
};
|
||||
|
||||
mod ctx;
|
||||
@ -117,7 +118,8 @@ pub(crate) struct VarUsageInfo {
|
||||
|
||||
pub pure_fn: bool,
|
||||
|
||||
/// In `c = b`, `b` infects `c`.
|
||||
/// `infects_to`. This should be renamed, but it will be done with another
|
||||
/// PR. (because it's hard to review)
|
||||
infects: Vec<Id>,
|
||||
}
|
||||
|
||||
@ -159,6 +161,39 @@ pub(crate) struct ProgramData {
|
||||
}
|
||||
|
||||
impl ProgramData {
|
||||
pub(crate) fn expand_infected(
|
||||
&self,
|
||||
ids: impl IntoIterator<Item = Id>,
|
||||
max_num: usize,
|
||||
) -> Result<FxHashSet<Id>, ()> {
|
||||
let mut result = FxHashSet::default();
|
||||
self.expand_infected_inner(ids, max_num, &mut result)?;
|
||||
Ok(result)
|
||||
}
|
||||
|
||||
fn expand_infected_inner(
|
||||
&self,
|
||||
ids: impl IntoIterator<Item = Id>,
|
||||
max_num: usize,
|
||||
result: &mut FxHashSet<Id>,
|
||||
) -> Result<(), ()> {
|
||||
for id in ids {
|
||||
if !result.insert(id.clone()) {
|
||||
continue;
|
||||
}
|
||||
if result.len() >= max_num {
|
||||
return Err(());
|
||||
}
|
||||
|
||||
if let Some(info) = self.vars.get(&id) {
|
||||
let ids = info.infects.clone();
|
||||
self.expand_infected_inner(ids, max_num, result)?;
|
||||
}
|
||||
}
|
||||
|
||||
Ok(())
|
||||
}
|
||||
|
||||
pub(crate) fn contains_unresolved(&self, e: &Expr) -> bool {
|
||||
match e {
|
||||
Expr::Ident(i) => {
|
||||
@ -603,16 +638,32 @@ where
|
||||
}
|
||||
|
||||
n.visit_children_with(self);
|
||||
|
||||
{
|
||||
for id in get_infects_of(&n.function) {
|
||||
self.data
|
||||
.var_or_default(n.ident.to_id())
|
||||
.add_infects_to(id.clone());
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
#[cfg_attr(feature = "debug", tracing::instrument(skip(self, n)))]
|
||||
fn visit_fn_expr(&mut self, n: &FnExpr) {
|
||||
n.visit_children_with(self);
|
||||
|
||||
if let Some(id) = &n.ident {
|
||||
if let Some(n_id) = &n.ident {
|
||||
self.data
|
||||
.var_or_default(id.to_id())
|
||||
.var_or_default(n_id.to_id())
|
||||
.mark_declared_as_fn_expr();
|
||||
|
||||
{
|
||||
for id in get_infects_of(&n.function) {
|
||||
self.data
|
||||
.var_or_default(n_id.to_id())
|
||||
.add_infects_to(id.to_id());
|
||||
}
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
@ -966,15 +1017,12 @@ where
|
||||
|
||||
for decl in &n.decls {
|
||||
if let (Pat::Ident(var), Some(init)) = (&decl.name, decl.init.as_deref()) {
|
||||
let used_idents = idents_used_by(init);
|
||||
let excluded: AHashSet<Id> = collect_decls(init);
|
||||
|
||||
for id in used_idents.into_iter().filter(|id| !excluded.contains(id)) {
|
||||
for id in get_infects_of(init) {
|
||||
self.data
|
||||
.var_or_default(id.clone())
|
||||
.add_infects(var.to_id());
|
||||
.add_infects_to(var.to_id());
|
||||
|
||||
self.data.var_or_default(var.to_id()).add_infects(id);
|
||||
self.data.var_or_default(var.to_id()).add_infects_to(id);
|
||||
}
|
||||
}
|
||||
}
|
||||
@ -1043,3 +1091,15 @@ fn is_safe_to_access_prop(e: &Expr) -> bool {
|
||||
_ => false,
|
||||
}
|
||||
}
|
||||
|
||||
fn get_infects_of<N>(init: &N) -> impl 'static + Iterator<Item = Id>
|
||||
where
|
||||
N: VisitWith<IdentUsageCollector> + VisitWith<BindingCollector<Id>>,
|
||||
{
|
||||
let used_idents = idents_used_by(init);
|
||||
let excluded: AHashSet<Id> = collect_decls(init);
|
||||
|
||||
used_idents
|
||||
.into_iter()
|
||||
.filter(move |id| !excluded.contains(id))
|
||||
}
|
||||
|
@ -61,7 +61,7 @@ pub(crate) trait VarDataLike: Sized {
|
||||
fn mark_mutated(&mut self);
|
||||
fn mark_reassigned_with_assign(&mut self);
|
||||
|
||||
fn add_infects(&mut self, other: Id);
|
||||
fn add_infects_to(&mut self, other: Id);
|
||||
|
||||
fn prevent_inline(&mut self);
|
||||
|
||||
|
@ -268,7 +268,7 @@ impl VarDataLike for VarUsageInfo {
|
||||
self.reassigned_with_assignment = true;
|
||||
}
|
||||
|
||||
fn add_infects(&mut self, other: Id) {
|
||||
fn add_infects_to(&mut self, other: Id) {
|
||||
self.infects.push(other);
|
||||
}
|
||||
|
||||
|
@ -13,6 +13,7 @@ use tracing::{span, Level};
|
||||
|
||||
use super::{is_pure_undefined, Optimizer};
|
||||
use crate::{
|
||||
alias::{collect_infects_from, AliasConfig},
|
||||
compress::{
|
||||
optimize::util::replace_id_with_expr,
|
||||
util::{is_directive, is_ident_used_by, replace_expr},
|
||||
@ -932,12 +933,14 @@ where
|
||||
return false;
|
||||
}
|
||||
|
||||
trace_op!("is_skippable_for_seq");
|
||||
|
||||
match e {
|
||||
Expr::Ident(e) => {
|
||||
if let Some(a) = a {
|
||||
match a {
|
||||
Mergable::Var(a) => {
|
||||
if is_ident_used_by(e.to_id(), &**a) {
|
||||
if is_ident_used_by(e.to_id(), &a.init) {
|
||||
log_abort!("ident used by a (var)");
|
||||
return false;
|
||||
}
|
||||
@ -949,6 +952,62 @@ where
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
// We can't proceed if the rhs (a.id = b.right) is
|
||||
// initialized with an initializer
|
||||
// (a.right) which has a side effect for pc (b.left)
|
||||
//
|
||||
// ```js
|
||||
//
|
||||
// function f(x) {
|
||||
// pc = 200;
|
||||
// return 100;
|
||||
// }
|
||||
// function x() {
|
||||
// var t = f();
|
||||
// pc += t;
|
||||
// return pc;
|
||||
// }
|
||||
// var pc = 0;
|
||||
// console.log(x());
|
||||
// ```
|
||||
//
|
||||
let ids_used_by_a_init = match a {
|
||||
Mergable::Var(a) => a.init.as_ref().map(|init| {
|
||||
collect_infects_from(init, AliasConfig { marks: self.marks })
|
||||
}),
|
||||
Mergable::Expr(a) => match a {
|
||||
Expr::Assign(AssignExpr {
|
||||
left,
|
||||
right,
|
||||
op: op!("="),
|
||||
..
|
||||
}) => {
|
||||
if left.as_ident().is_some() {
|
||||
Some(collect_infects_from(
|
||||
right,
|
||||
AliasConfig { marks: self.marks },
|
||||
))
|
||||
} else {
|
||||
None
|
||||
}
|
||||
}
|
||||
|
||||
_ => None,
|
||||
},
|
||||
};
|
||||
|
||||
if let Some(ids_used_by_a_init) = ids_used_by_a_init {
|
||||
let deps = self.data.expand_infected(ids_used_by_a_init, 64);
|
||||
|
||||
let deps = match deps {
|
||||
Ok(v) => v,
|
||||
Err(()) => return false,
|
||||
};
|
||||
if deps.contains(&e.to_id()) {
|
||||
return false;
|
||||
}
|
||||
}
|
||||
}
|
||||
|
||||
return true;
|
||||
@ -1240,7 +1299,7 @@ where
|
||||
},
|
||||
}
|
||||
|
||||
if should_not_check_rhs_of_assign(a, b) {
|
||||
if self.should_not_check_rhs_of_assign(a, b)? {
|
||||
return Ok(false);
|
||||
}
|
||||
|
||||
@ -1249,7 +1308,7 @@ where
|
||||
}
|
||||
|
||||
Expr::Assign(b) => {
|
||||
if should_not_check_rhs_of_assign(a, b) {
|
||||
if self.should_not_check_rhs_of_assign(a, b)? {
|
||||
return Ok(false);
|
||||
}
|
||||
|
||||
@ -1259,6 +1318,10 @@ where
|
||||
None => return Ok(false),
|
||||
};
|
||||
|
||||
if !self.is_skippable_for_seq(Some(a), &Expr::Ident(b_left.clone())) {
|
||||
return Ok(false);
|
||||
}
|
||||
|
||||
if UsageFinder::find(&b_left, &b.right) {
|
||||
return Err(());
|
||||
}
|
||||
@ -1661,12 +1724,12 @@ where
|
||||
|
||||
let used_by_b = idents_used_by(&*b);
|
||||
|
||||
for id in &deps {
|
||||
if *id == left_id.to_id() {
|
||||
for dep_id in &deps {
|
||||
if *dep_id == left_id.to_id() {
|
||||
continue;
|
||||
}
|
||||
|
||||
if used_by_b.contains(id) {
|
||||
if used_by_b.contains(dep_id) {
|
||||
log_abort!("[X] sequences: Aborting because of deps");
|
||||
return Err(());
|
||||
}
|
||||
@ -1712,31 +1775,32 @@ where
|
||||
|
||||
Ok(true)
|
||||
}
|
||||
}
|
||||
|
||||
/// TODO(kdy1): Optimize this
|
||||
///
|
||||
/// See https://github.com/swc-project/swc/pull/3480
|
||||
///
|
||||
/// This works, but it should be optimized.
|
||||
///
|
||||
/// This check blocks optimization of clearly valid optimizations like `i += 1,
|
||||
/// arr[i]`
|
||||
fn should_not_check_rhs_of_assign(a: &Mergable, b: &mut AssignExpr) -> bool {
|
||||
if let Some(a_id) = a.id() {
|
||||
match a {
|
||||
Mergable::Expr(Expr::Assign(AssignExpr { op: op!("="), .. })) => {}
|
||||
Mergable::Expr(Expr::Assign(..)) => {
|
||||
let used_by_b = idents_used_by(&*b.right);
|
||||
if used_by_b.contains(&a_id) {
|
||||
return true;
|
||||
/// TODO(kdy1): Optimize this
|
||||
///
|
||||
/// See https://github.com/swc-project/swc/pull/3480
|
||||
///
|
||||
/// This works, but it should be optimized.
|
||||
///
|
||||
/// This check blocks optimization of clearly valid optimizations like `i +=
|
||||
/// 1, arr[i]`
|
||||
//
|
||||
fn should_not_check_rhs_of_assign(&self, a: &Mergable, b: &mut AssignExpr) -> Result<bool, ()> {
|
||||
if let Some(a_id) = a.id() {
|
||||
match a {
|
||||
Mergable::Expr(Expr::Assign(AssignExpr { op: op!("="), .. })) => {}
|
||||
Mergable::Expr(Expr::Assign(..)) => {
|
||||
let used_by_b = idents_used_by(&*b.right);
|
||||
if used_by_b.contains(&a_id) {
|
||||
return Ok(true);
|
||||
}
|
||||
}
|
||||
_ => {}
|
||||
}
|
||||
_ => {}
|
||||
}
|
||||
}
|
||||
|
||||
false
|
||||
Ok(false)
|
||||
}
|
||||
}
|
||||
|
||||
struct UsageCounter<'a> {
|
||||
|
@ -50,6 +50,7 @@ use crate::{
|
||||
|
||||
#[macro_use]
|
||||
mod macros;
|
||||
mod alias;
|
||||
mod analyzer;
|
||||
mod compress;
|
||||
mod debug;
|
||||
|
@ -1,8 +1,8 @@
|
||||
use std::time::Instant;
|
||||
|
||||
use rustc_hash::FxHashSet;
|
||||
use swc_atoms::js_word;
|
||||
use swc_common::{
|
||||
collections::AHashSet,
|
||||
pass::{CompilerPass, Repeated},
|
||||
util::take::Take,
|
||||
Mark, Span, Spanned, DUMMY_SP,
|
||||
@ -379,7 +379,7 @@ where
|
||||
|
||||
#[derive(Default)]
|
||||
pub(crate) struct IdentUsageCollector {
|
||||
ids: AHashSet<Id>,
|
||||
ids: FxHashSet<Id>,
|
||||
ignore_nested: bool,
|
||||
}
|
||||
|
||||
@ -425,7 +425,7 @@ impl Visit for IdentUsageCollector {
|
||||
|
||||
#[derive(Default)]
|
||||
pub(crate) struct CapturedIdCollector {
|
||||
ids: AHashSet<Id>,
|
||||
ids: FxHashSet<Id>,
|
||||
is_nested: bool,
|
||||
}
|
||||
|
||||
@ -468,7 +468,7 @@ impl Visit for CapturedIdCollector {
|
||||
}
|
||||
}
|
||||
|
||||
pub(crate) fn idents_captured_by<N>(n: &N) -> AHashSet<Id>
|
||||
pub(crate) fn idents_captured_by<N>(n: &N) -> FxHashSet<Id>
|
||||
where
|
||||
N: VisitWith<CapturedIdCollector>,
|
||||
{
|
||||
@ -480,7 +480,7 @@ where
|
||||
v.ids
|
||||
}
|
||||
|
||||
pub(crate) fn idents_used_by<N>(n: &N) -> AHashSet<Id>
|
||||
pub(crate) fn idents_used_by<N>(n: &N) -> FxHashSet<Id>
|
||||
where
|
||||
N: VisitWith<IdentUsageCollector>,
|
||||
{
|
||||
@ -492,7 +492,7 @@ where
|
||||
v.ids
|
||||
}
|
||||
|
||||
pub(crate) fn idents_used_by_ignoring_nested<N>(n: &N) -> AHashSet<Id>
|
||||
pub(crate) fn idents_used_by_ignoring_nested<N>(n: &N) -> FxHashSet<Id>
|
||||
where
|
||||
N: VisitWith<IdentUsageCollector>,
|
||||
{
|
||||
|
@ -9,9 +9,6 @@ collapse_vars/collapse_vars_side_effects_1/input.js
|
||||
collapse_vars/collapse_vars_side_effects_2/input.js
|
||||
collapse_vars/collapse_vars_switch/input.js
|
||||
collapse_vars/collapse_vars_unary/input.js
|
||||
collapse_vars/issue_1631_1/input.js
|
||||
collapse_vars/issue_1631_2/input.js
|
||||
collapse_vars/issue_1631_3/input.js
|
||||
collapse_vars/issue_2436_10/input.js
|
||||
collapse_vars/issue_2436_11/input.js
|
||||
collapse_vars/issue_2436_9/input.js
|
||||
|
@ -46593,7 +46593,7 @@ TestSnapshot {
|
||||
declared_count: 0,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 3,
|
||||
assign_count: 5,
|
||||
mutation_by_call_count: 7,
|
||||
usage_count: 271,
|
||||
reassigned_with_assignment: false,
|
||||
@ -121105,7 +121105,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 3,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 1,
|
||||
reassigned_with_assignment: true,
|
||||
@ -138935,12 +138935,12 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: false,
|
||||
reassigned_with_var_decl: false,
|
||||
mutated: false,
|
||||
mutated: true,
|
||||
has_property_access: true,
|
||||
has_property_mutation: false,
|
||||
accessed_props: {},
|
||||
@ -222401,7 +222401,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: true,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 3,
|
||||
reassigned_with_assignment: false,
|
||||
|
@ -327,7 +327,10 @@
|
||||
var tmp = appConfig.request, requestConfig = void 0 === tmp ? {} : tmp;
|
||||
"[object Array]" === Object.prototype.toString.call(requestConfig) ? requestConfig.forEach(function(requestItem) {
|
||||
var instanceName = requestItem.instanceName ? requestItem.instanceName : "default";
|
||||
instanceName && setAxiosInstance(requestItem, _createAxiosInstance.default(instanceName)[instanceName]);
|
||||
if (instanceName) {
|
||||
var axiosInstance = _createAxiosInstance.default(instanceName)[instanceName];
|
||||
setAxiosInstance(requestItem, axiosInstance);
|
||||
}
|
||||
}) : setAxiosInstance(requestConfig, _createAxiosInstance.default().default);
|
||||
}
|
||||
};
|
||||
@ -352,7 +355,9 @@
|
||||
return _formatRoutes.default(appConfigRouter.routes || _routes.default, "");
|
||||
}), modifyRoutesComponent(function() {
|
||||
return _router.Routes;
|
||||
}), wrapperPageComponent(process.env.__IS_SERVER__ ? _formatRoutes.wrapperPageWithSSR(context) : _formatRoutes.wrapperPageWithCSR()), wrapperPageComponent(function(PageComponent) {
|
||||
});
|
||||
var wrapperPageFn = process.env.__IS_SERVER__ ? _formatRoutes.wrapperPageWithSSR(context) : _formatRoutes.wrapperPageWithCSR();
|
||||
wrapperPageComponent(wrapperPageFn), wrapperPageComponent(function(PageComponent) {
|
||||
var _pageConfig = PageComponent.pageConfig, pageConfig = void 0 === _pageConfig ? {} : _pageConfig;
|
||||
return function(props) {
|
||||
return pageConfig.errorBoundary ? _jsxRuntime.jsx(_errorBoundary.default, {
|
||||
@ -745,13 +750,13 @@
|
||||
} : _ref$defaultResolveCo, _render = _ref.render, onLoad = _ref.onLoad;
|
||||
function loadable(loadableConstructor, options) {
|
||||
void 0 === options && (options = {});
|
||||
var ctor = "function" == typeof (ctor1 = loadableConstructor) ? {
|
||||
requireAsync: ctor1,
|
||||
var ctor, ctor1 = "function" == typeof (ctor = loadableConstructor) ? {
|
||||
requireAsync: ctor,
|
||||
resolve: function() {},
|
||||
chunkName: function() {}
|
||||
} : ctor1, cache = {};
|
||||
} : ctor, cache = {};
|
||||
function _getCacheKey(props) {
|
||||
return options.cacheKey ? options.cacheKey(props) : ctor.resolve ? ctor.resolve(props) : "static";
|
||||
return options.cacheKey ? options.cacheKey(props) : ctor1.resolve ? ctor1.resolve(props) : "static";
|
||||
}
|
||||
function resolve(module, props, Loadable) {
|
||||
var Component = options.resolveComponent ? options.resolveComponent(module, props) : defaultResolveComponent(module);
|
||||
@ -760,7 +765,7 @@
|
||||
preload: !0
|
||||
}), Component;
|
||||
}
|
||||
var ctor1, EnhancedInnerLoadable = withChunkExtractor(function(_React$Component) {
|
||||
var InnerLoadable1 = function(_React$Component) {
|
||||
function InnerLoadable(props) {
|
||||
var _this;
|
||||
return ((_this = _React$Component.call(this, props) || this).state = {
|
||||
@ -768,12 +773,12 @@
|
||||
error: null,
|
||||
loading: !0,
|
||||
cacheKey: _getCacheKey(props)
|
||||
}, invariant(!props.__chunkExtractor || ctor.requireSync, "SSR requires `@loadable/babel-plugin`, please install it"), props.__chunkExtractor) ? (!1 === options.ssr || (ctor.requireAsync(props).catch(function() {
|
||||
}, invariant(!props.__chunkExtractor || ctor1.requireSync, "SSR requires `@loadable/babel-plugin`, please install it"), props.__chunkExtractor) ? (!1 === options.ssr || (ctor1.requireAsync(props).catch(function() {
|
||||
return null;
|
||||
}), _this.loadSync(), props.__chunkExtractor.addChunk(ctor.chunkName(props))), function(self) {
|
||||
}), _this.loadSync(), props.__chunkExtractor.addChunk(ctor1.chunkName(props))), function(self) {
|
||||
if (void 0 === self) throw new ReferenceError("this hasn't been initialised - super() hasn't been called");
|
||||
return self;
|
||||
}(_this)) : (!1 !== options.ssr && (ctor.isReady && ctor.isReady(props) || ctor.chunkName && LOADABLE_SHARED.initialChunks[ctor.chunkName(props)]) && _this.loadSync(), _this);
|
||||
}(_this)) : (!1 !== options.ssr && (ctor1.isReady && ctor1.isReady(props) || ctor1.chunkName && LOADABLE_SHARED.initialChunks[ctor1.chunkName(props)]) && _this.loadSync(), _this);
|
||||
}
|
||||
(0, inheritsLoose.Z)(InnerLoadable, _React$Component), InnerLoadable.getDerivedStateFromProps = function(props, state) {
|
||||
var cacheKey = _getCacheKey(props);
|
||||
@ -806,12 +811,12 @@
|
||||
});
|
||||
}, _proto.loadSync = function() {
|
||||
if (this.state.loading) try {
|
||||
var loadedModule = ctor.requireSync(this.props), result = resolve(loadedModule, this.props, Loadable1);
|
||||
var loadedModule = ctor1.requireSync(this.props), result = resolve(loadedModule, this.props, Loadable1);
|
||||
this.state.result = result, this.state.loading = !1;
|
||||
} catch (error) {
|
||||
console.error("loadable-components: failed to synchronously load component, which expected to be available", {
|
||||
fileName: ctor.resolve(this.props),
|
||||
chunkName: ctor.chunkName(this.props),
|
||||
fileName: ctor1.resolve(this.props),
|
||||
chunkName: ctor1.chunkName(this.props),
|
||||
error: error ? error.message : error
|
||||
}), this.state.error = error;
|
||||
}
|
||||
@ -838,12 +843,12 @@
|
||||
"__chunkExtractor",
|
||||
"forwardedRef"
|
||||
])), promise = this.getCache();
|
||||
return promise || ((promise = ctor.requireAsync(props)).status = STATUS_PENDING, this.setCache(promise), promise.then(function() {
|
||||
return promise || ((promise = ctor1.requireAsync(props)).status = STATUS_PENDING, this.setCache(promise), promise.then(function() {
|
||||
promise.status = "RESOLVED";
|
||||
}, function(error) {
|
||||
console.error("loadable-components: failed to asynchronously load component", {
|
||||
fileName: ctor.resolve(_this4.props),
|
||||
chunkName: ctor.chunkName(_this4.props),
|
||||
fileName: ctor1.resolve(_this4.props),
|
||||
chunkName: ctor1.chunkName(_this4.props),
|
||||
error: error ? error.message : error
|
||||
}), promise.status = STATUS_REJECTED;
|
||||
})), promise;
|
||||
@ -865,15 +870,15 @@
|
||||
})
|
||||
});
|
||||
}, InnerLoadable;
|
||||
}(_react_17_0_2_react.Component)), Loadable1 = _react_17_0_2_react.forwardRef(function(props, ref) {
|
||||
}(_react_17_0_2_react.Component), EnhancedInnerLoadable = withChunkExtractor(InnerLoadable1), Loadable1 = _react_17_0_2_react.forwardRef(function(props, ref) {
|
||||
return _react_17_0_2_react.createElement(EnhancedInnerLoadable, Object.assign({
|
||||
forwardedRef: ref
|
||||
}, props));
|
||||
});
|
||||
return Loadable1.displayName = "Loadable", Loadable1.preload = function(props) {
|
||||
ctor.requireAsync(props);
|
||||
ctor1.requireAsync(props);
|
||||
}, Loadable1.load = function(props) {
|
||||
return ctor.requireAsync(props);
|
||||
return ctor1.requireAsync(props);
|
||||
}, Loadable1;
|
||||
}
|
||||
return {
|
||||
@ -1021,11 +1026,11 @@
|
||||
function _asyncGeneratorDelegate(inner, awaitWrap) {
|
||||
var iter = {}, waiting = !1;
|
||||
function pump(key, value) {
|
||||
return waiting = !0, {
|
||||
return waiting = !0, value = new Promise(function(resolve) {
|
||||
resolve(inner[key](value));
|
||||
}), {
|
||||
done: !1,
|
||||
value: awaitWrap(value = new Promise(function(resolve) {
|
||||
resolve(inner[key](value));
|
||||
}))
|
||||
value: awaitWrap(value)
|
||||
};
|
||||
}
|
||||
return "function" == typeof Symbol && Symbol.iterator && (iter[Symbol.iterator] = function() {
|
||||
@ -1378,9 +1383,9 @@
|
||||
var kind = String(obj.kind);
|
||||
if ("class" !== kind) throw new TypeError('A class descriptor\'s .kind property must be "class", but a decorator created a class descriptor with .kind "' + kind + '"');
|
||||
_disallowProperty(obj, "key", "A class descriptor"), _disallowProperty(obj, "placement", "A class descriptor"), _disallowProperty(obj, "descriptor", "A class descriptor"), _disallowProperty(obj, "initializer", "A class descriptor"), _disallowProperty(obj, "extras", "A class descriptor");
|
||||
var finisher = _optionalCallableProperty(obj, "finisher"), elements = _toElementDescriptors(obj.elements);
|
||||
var finisher = _optionalCallableProperty(obj, "finisher");
|
||||
return {
|
||||
elements: elements,
|
||||
elements: _toElementDescriptors(obj.elements),
|
||||
finisher: finisher
|
||||
};
|
||||
}
|
||||
@ -1941,15 +1946,15 @@
|
||||
var fullPath = buildFullPath(config.baseURL, config.url);
|
||||
function onloadend() {
|
||||
if (request) {
|
||||
var responseHeaders = "getAllResponseHeaders" in request ? parseHeaders(request.getAllResponseHeaders()) : null;
|
||||
settle(resolve, reject, {
|
||||
var responseHeaders = "getAllResponseHeaders" in request ? parseHeaders(request.getAllResponseHeaders()) : null, response = {
|
||||
data: responseType && "text" !== responseType && "json" !== responseType ? request.response : request.responseText,
|
||||
status: request.status,
|
||||
statusText: request.statusText,
|
||||
headers: responseHeaders,
|
||||
config: config,
|
||||
request: request
|
||||
}), request = null;
|
||||
};
|
||||
settle(resolve, reject, response), request = null;
|
||||
}
|
||||
}
|
||||
if (request.open(config.method.toUpperCase(), buildURL(fullPath, config.params, config.paramsSerializer), !0), request.timeout = config.timeout, "onloadend" in request ? request.onloadend = onloadend : request.onreadystatechange = function() {
|
||||
@ -2076,7 +2081,7 @@
|
||||
for(; responseInterceptorChain.length;)promise = promise.then(responseInterceptorChain.shift(), responseInterceptorChain.shift());
|
||||
return promise;
|
||||
}, Axios.prototype.getUri = function(config) {
|
||||
return buildURL((config = mergeConfig(this.defaults, config)).url, config.params, config.paramsSerializer).replace(/^\?/, "");
|
||||
return config = mergeConfig(this.defaults, config), buildURL(config.url, config.params, config.paramsSerializer).replace(/^\?/, "");
|
||||
}, utils.forEach([
|
||||
"delete",
|
||||
"get",
|
||||
@ -2136,7 +2141,8 @@
|
||||
"use strict";
|
||||
var enhanceError = __webpack_require__(16488);
|
||||
module.exports = function(message, config, code, request, response) {
|
||||
return enhanceError(new Error(message), config, code, request, response);
|
||||
var error = new Error(message);
|
||||
return enhanceError(error, config, code, request, response);
|
||||
};
|
||||
},
|
||||
41388: function(module, __unused_webpack_exports, __webpack_require__) {
|
||||
@ -3627,9 +3633,9 @@
|
||||
35437: function(module, __unused_webpack_exports, __webpack_require__) {
|
||||
var global = __webpack_require__(19514), getOwnPropertyDescriptor = __webpack_require__(24722).f, createNonEnumerableProperty = __webpack_require__(48181), redefine = __webpack_require__(78109), setGlobal = __webpack_require__(65933), copyConstructorProperties = __webpack_require__(18295), isForced = __webpack_require__(23736);
|
||||
module.exports = function(options, source) {
|
||||
var FORCED, target, key, targetProperty, sourceProperty, descriptor, TARGET = options.target, GLOBAL = options.global, STATIC = options.stat;
|
||||
var target, key, targetProperty, sourceProperty, descriptor, TARGET = options.target, GLOBAL = options.global, STATIC = options.stat;
|
||||
if (target = GLOBAL ? global : STATIC ? global[TARGET] || setGlobal(TARGET, {}) : (global[TARGET] || {}).prototype) for(key in source){
|
||||
if (sourceProperty = source[key], targetProperty = options.noTargetGet ? (descriptor = getOwnPropertyDescriptor(target, key)) && descriptor.value : target[key], FORCED = isForced(GLOBAL ? key : TARGET + (STATIC ? "." : "#") + key, options.forced), !FORCED && void 0 !== targetProperty) {
|
||||
if (sourceProperty = source[key], targetProperty = options.noTargetGet ? (descriptor = getOwnPropertyDescriptor(target, key)) && descriptor.value : target[key], !isForced(GLOBAL ? key : TARGET + (STATIC ? "." : "#") + key, options.forced) && void 0 !== targetProperty) {
|
||||
if (typeof sourceProperty == typeof targetProperty) continue;
|
||||
copyConstructorProperties(sourceProperty, targetProperty);
|
||||
}
|
||||
@ -4864,7 +4870,7 @@
|
||||
if (!isObject(input) || isSymbol(input)) return input;
|
||||
var result, exoticToPrim = getMethod(input, TO_PRIMITIVE);
|
||||
if (exoticToPrim) {
|
||||
if (void 0 === pref && (pref = "default"), !isObject(result = exoticToPrim.call(input, pref)) || isSymbol(result)) return result;
|
||||
if (void 0 === pref && (pref = "default"), result = exoticToPrim.call(input, pref), !isObject(result) || isSymbol(result)) return result;
|
||||
throw TypeError("Can't convert object to primitive value");
|
||||
}
|
||||
return void 0 === pref && (pref = "number"), ordinaryToPrimitive(input, pref);
|
||||
@ -4914,9 +4920,9 @@
|
||||
}, isTypedArrayIndex = function(target, key) {
|
||||
return isTypedArray(target) && !isSymbol(key) && key in target && isInteger(+key) && key >= 0;
|
||||
}, wrappedGetOwnPropertyDescriptor = function(target, key) {
|
||||
return isTypedArrayIndex(target, key = toPropertyKey(key)) ? createPropertyDescriptor(2, target[key]) : nativeGetOwnPropertyDescriptor(target, key);
|
||||
return key = toPropertyKey(key), isTypedArrayIndex(target, key) ? createPropertyDescriptor(2, target[key]) : nativeGetOwnPropertyDescriptor(target, key);
|
||||
}, wrappedDefineProperty = function(target, key, descriptor) {
|
||||
return isTypedArrayIndex(target, key = toPropertyKey(key)) && isObject(descriptor) && has(descriptor, "value") && !has(descriptor, "get") && !has(descriptor, "set") && !descriptor.configurable && (!has(descriptor, "writable") || descriptor.writable) && (!has(descriptor, "enumerable") || descriptor.enumerable) ? (target[key] = descriptor.value, target) : nativeDefineProperty(target, key, descriptor);
|
||||
return (key = toPropertyKey(key), isTypedArrayIndex(target, key) && isObject(descriptor) && has(descriptor, "value") && !has(descriptor, "get") && !has(descriptor, "set") && !descriptor.configurable && (!has(descriptor, "writable") || descriptor.writable) && (!has(descriptor, "enumerable") || descriptor.enumerable)) ? (target[key] = descriptor.value, target) : nativeDefineProperty(target, key, descriptor);
|
||||
};
|
||||
DESCRIPTORS ? (NATIVE_ARRAY_BUFFER_VIEWS || (getOwnPropertyDescriptorModule.f = wrappedGetOwnPropertyDescriptor, definePropertyModule.f = wrappedDefineProperty, addGetter(TypedArrayPrototype, "buffer"), addGetter(TypedArrayPrototype, "byteOffset"), addGetter(TypedArrayPrototype, "byteLength"), addGetter(TypedArrayPrototype, "length")), $({
|
||||
target: "Object",
|
||||
@ -5809,11 +5815,11 @@
|
||||
});
|
||||
},
|
||||
50241: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
var $ = __webpack_require__(35437), $hypot = Math.hypot, abs = Math.abs, sqrt = Math.sqrt;
|
||||
var $ = __webpack_require__(35437), $hypot = Math.hypot, abs = Math.abs, sqrt = Math.sqrt, BUGGY = !!$hypot && $hypot(1 / 0, NaN) !== 1 / 0;
|
||||
$({
|
||||
target: "Math",
|
||||
stat: !0,
|
||||
forced: !!$hypot && $hypot(1 / 0, NaN) !== 1 / 0
|
||||
forced: BUGGY
|
||||
}, {
|
||||
hypot: function(value1, value2) {
|
||||
for(var arg, div, sum = 0, i = 0, aLen = arguments.length, larg = 0; i < aLen;)arg = abs(arguments[i++]), larg < arg ? (sum = sum * (div = larg / arg) * div + 1, larg = arg) : arg > 0 ? sum += (div = arg / larg) * div : sum += arg;
|
||||
@ -6932,15 +6938,16 @@
|
||||
}
|
||||
return !0;
|
||||
}
|
||||
var MS_EDGE_BUG = fails(function() {
|
||||
var Constructor = function() {}, object = definePropertyModule.f(new Constructor(), "a", {
|
||||
configurable: !0
|
||||
});
|
||||
return !1 !== Reflect.set(Constructor.prototype, "a", 1, object);
|
||||
});
|
||||
$({
|
||||
target: "Reflect",
|
||||
stat: !0,
|
||||
forced: fails(function() {
|
||||
var Constructor = function() {}, object = definePropertyModule.f(new Constructor(), "a", {
|
||||
configurable: !0
|
||||
});
|
||||
return !1 !== Reflect.set(Constructor.prototype, "a", 1, object);
|
||||
})
|
||||
forced: MS_EDGE_BUG
|
||||
}, {
|
||||
set: set
|
||||
});
|
||||
@ -7459,7 +7466,15 @@
|
||||
},
|
||||
54878: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
"use strict";
|
||||
var fixRegExpWellKnownSymbolLogic = __webpack_require__(29045), fails = __webpack_require__(60232), anObject = __webpack_require__(83941), isCallable = __webpack_require__(67106), toInteger = __webpack_require__(86361), toLength = __webpack_require__(31998), toString = __webpack_require__(72729), requireObjectCoercible = __webpack_require__(79602), advanceStringIndex = __webpack_require__(88770), getMethod = __webpack_require__(84316), getSubstitution = __webpack_require__(33371), regExpExec = __webpack_require__(21135), wellKnownSymbol = __webpack_require__(81019), REPLACE = wellKnownSymbol("replace"), max = Math.max, min = Math.min, REPLACE_KEEPS_$0 = "$0" === "a".replace(/./, "$0"), REGEXP_REPLACE_SUBSTITUTES_UNDEFINED_CAPTURE = !!/./[REPLACE] && "" === /./[REPLACE]("a", "$0");
|
||||
var fixRegExpWellKnownSymbolLogic = __webpack_require__(29045), fails = __webpack_require__(60232), anObject = __webpack_require__(83941), isCallable = __webpack_require__(67106), toInteger = __webpack_require__(86361), toLength = __webpack_require__(31998), toString = __webpack_require__(72729), requireObjectCoercible = __webpack_require__(79602), advanceStringIndex = __webpack_require__(88770), getMethod = __webpack_require__(84316), getSubstitution = __webpack_require__(33371), regExpExec = __webpack_require__(21135), wellKnownSymbol = __webpack_require__(81019), REPLACE = wellKnownSymbol("replace"), max = Math.max, min = Math.min, REPLACE_KEEPS_$0 = "$0" === "a".replace(/./, "$0"), REGEXP_REPLACE_SUBSTITUTES_UNDEFINED_CAPTURE = !!/./[REPLACE] && "" === /./[REPLACE]("a", "$0"), REPLACE_SUPPORTS_NAMED_GROUPS = !fails(function() {
|
||||
var re = /./;
|
||||
return re.exec = function() {
|
||||
var result = [];
|
||||
return result.groups = {
|
||||
a: "7"
|
||||
}, result;
|
||||
}, "7" !== "".replace(re, "$<a>");
|
||||
});
|
||||
fixRegExpWellKnownSymbolLogic("replace", function(_, nativeReplace, maybeCallNative) {
|
||||
var UNSAFE_SUBSTITUTE = REGEXP_REPLACE_SUBSTITUTES_UNDEFINED_CAPTURE ? "$" : "$0";
|
||||
return [
|
||||
@ -7501,15 +7516,7 @@
|
||||
return accumulatedResult + S.slice(nextSourcePosition);
|
||||
},
|
||||
];
|
||||
}, !!fails(function() {
|
||||
var re = /./;
|
||||
return re.exec = function() {
|
||||
var result = [];
|
||||
return result.groups = {
|
||||
a: "7"
|
||||
}, result;
|
||||
}, "7" !== "".replace(re, "$<a>");
|
||||
}) || !REPLACE_KEEPS_$0 || REGEXP_REPLACE_SUBSTITUTES_UNDEFINED_CAPTURE);
|
||||
}, !REPLACE_SUPPORTS_NAMED_GROUPS || !REPLACE_KEEPS_$0 || REGEXP_REPLACE_SUBSTITUTES_UNDEFINED_CAPTURE);
|
||||
},
|
||||
49000: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
"use strict";
|
||||
@ -7546,7 +7553,14 @@
|
||||
},
|
||||
1752: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
"use strict";
|
||||
var fixRegExpWellKnownSymbolLogic = __webpack_require__(29045), isRegExp = __webpack_require__(78202), anObject = __webpack_require__(83941), requireObjectCoercible = __webpack_require__(79602), speciesConstructor = __webpack_require__(94850), advanceStringIndex = __webpack_require__(88770), toLength = __webpack_require__(31998), toString = __webpack_require__(72729), getMethod = __webpack_require__(84316), callRegExpExec = __webpack_require__(21135), regexpExec = __webpack_require__(72384), stickyHelpers = __webpack_require__(44725), fails = __webpack_require__(60232), UNSUPPORTED_Y = stickyHelpers.UNSUPPORTED_Y, arrayPush = [].push, min = Math.min;
|
||||
var fixRegExpWellKnownSymbolLogic = __webpack_require__(29045), isRegExp = __webpack_require__(78202), anObject = __webpack_require__(83941), requireObjectCoercible = __webpack_require__(79602), speciesConstructor = __webpack_require__(94850), advanceStringIndex = __webpack_require__(88770), toLength = __webpack_require__(31998), toString = __webpack_require__(72729), getMethod = __webpack_require__(84316), callRegExpExec = __webpack_require__(21135), regexpExec = __webpack_require__(72384), stickyHelpers = __webpack_require__(44725), fails = __webpack_require__(60232), UNSUPPORTED_Y = stickyHelpers.UNSUPPORTED_Y, arrayPush = [].push, min = Math.min, SPLIT_WORKS_WITH_OVERWRITTEN_EXEC = !fails(function() {
|
||||
var re = /(?:)/, originalExec = re.exec;
|
||||
re.exec = function() {
|
||||
return originalExec.apply(this, arguments);
|
||||
};
|
||||
var result = "ab".split(re);
|
||||
return 2 !== result.length || "a" !== result[0] || "b" !== result[1];
|
||||
});
|
||||
fixRegExpWellKnownSymbolLogic("split", function(SPLIT, nativeSplit, maybeCallNative) {
|
||||
var internalSplit;
|
||||
return internalSplit = "c" == "abbc".split(/(b)*/)[1] || 4 != "test".split(/(?:)/, -1).length || 2 != "ab".split(/(?:ab)*/).length || 4 != ".".split(/(.?)(.?)/).length || ".".split(/()()/).length > 1 || "".split(/.?/).length ? function(separator, limit) {
|
||||
@ -7586,14 +7600,7 @@
|
||||
return A.push(S.slice(p)), A;
|
||||
},
|
||||
];
|
||||
}, !!fails(function() {
|
||||
var re = /(?:)/, originalExec = re.exec;
|
||||
re.exec = function() {
|
||||
return originalExec.apply(this, arguments);
|
||||
};
|
||||
var result = "ab".split(re);
|
||||
return 2 !== result.length || "a" !== result[0] || "b" !== result[1];
|
||||
}), UNSUPPORTED_Y);
|
||||
}, !SPLIT_WORKS_WITH_OVERWRITTEN_EXEC, UNSUPPORTED_Y);
|
||||
},
|
||||
24467: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
"use strict";
|
||||
@ -7774,8 +7781,8 @@
|
||||
})) : (has(O, HIDDEN) || nativeDefineProperty(O, HIDDEN, createPropertyDescriptor(1, {})), O[HIDDEN][key] = !0), setSymbolDescriptor(O, key, Attributes)) : nativeDefineProperty(O, key, Attributes);
|
||||
}, $defineProperties = function(O, Properties) {
|
||||
anObject(O);
|
||||
var properties = toIndexedObject(Properties);
|
||||
return $forEach(objectKeys(properties).concat($getOwnPropertySymbols(properties)), function(key) {
|
||||
var properties = toIndexedObject(Properties), keys = objectKeys(properties).concat($getOwnPropertySymbols(properties));
|
||||
return $forEach(keys, function(key) {
|
||||
(!DESCRIPTORS || $propertyIsEnumerable.call(properties, key)) && $defineProperty(O, key, properties[key]);
|
||||
}), O;
|
||||
}, $propertyIsEnumerable = function(V) {
|
||||
@ -7798,7 +7805,7 @@
|
||||
has(AllSymbols, key) && (!IS_OBJECT_PROTOTYPE || has(ObjectPrototype, key)) && result.push(AllSymbols[key]);
|
||||
}), result;
|
||||
};
|
||||
if (NATIVE_SYMBOL || (redefine(($Symbol = function() {
|
||||
if (NATIVE_SYMBOL || ($Symbol = function() {
|
||||
if (this instanceof $Symbol) throw TypeError("Symbol is not a constructor");
|
||||
var description = arguments.length && void 0 !== arguments[0] ? $toString(arguments[0]) : void 0, tag = uid(description), setter = function(value) {
|
||||
this === ObjectPrototype && setter.call(ObjectPrototypeSymbols, value), has(this, HIDDEN) && has(this[HIDDEN], tag) && (this[HIDDEN][tag] = !1), setSymbolDescriptor(this, tag, createPropertyDescriptor(1, value));
|
||||
@ -7807,7 +7814,7 @@
|
||||
configurable: !0,
|
||||
set: setter
|
||||
}), wrap(tag, description);
|
||||
})[PROTOTYPE], "toString", function() {
|
||||
}, redefine($Symbol[PROTOTYPE], "toString", function() {
|
||||
return getInternalState(this).tag;
|
||||
}), redefine($Symbol, "withoutSetter", function(description) {
|
||||
return wrap(uid(description), description);
|
||||
@ -7879,27 +7886,31 @@
|
||||
getOwnPropertySymbols: function(it) {
|
||||
return getOwnPropertySymbolsModule.f(toObject(it));
|
||||
}
|
||||
}), $stringify && $({
|
||||
target: "JSON",
|
||||
stat: !0,
|
||||
forced: !NATIVE_SYMBOL || fails(function() {
|
||||
}), $stringify) {
|
||||
var FORCED_JSON_STRINGIFY = !NATIVE_SYMBOL || fails(function() {
|
||||
var symbol = $Symbol();
|
||||
return "[null]" != $stringify([
|
||||
symbol
|
||||
]) || "{}" != $stringify({
|
||||
a: symbol
|
||||
}) || "{}" != $stringify(Object(symbol));
|
||||
})
|
||||
}, {
|
||||
stringify: function(it, replacer, space) {
|
||||
for(var $replacer, args = [
|
||||
it
|
||||
], index = 1; arguments.length > index;)args.push(arguments[index++]);
|
||||
if ($replacer = replacer, !(!isObject(replacer) && void 0 === it || isSymbol(it))) return isArray(replacer) || (replacer = function(key, value) {
|
||||
if (isCallable($replacer) && (value = $replacer.call(this, key, value)), !isSymbol(value)) return value;
|
||||
}), args[1] = replacer, $stringify.apply(null, args);
|
||||
}
|
||||
}), !$Symbol[PROTOTYPE][TO_PRIMITIVE]) {
|
||||
});
|
||||
$({
|
||||
target: "JSON",
|
||||
stat: !0,
|
||||
forced: FORCED_JSON_STRINGIFY
|
||||
}, {
|
||||
stringify: function(it, replacer, space) {
|
||||
for(var $replacer, args = [
|
||||
it
|
||||
], index = 1; arguments.length > index;)args.push(arguments[index++]);
|
||||
if ($replacer = replacer, !(!isObject(replacer) && void 0 === it || isSymbol(it))) return isArray(replacer) || (replacer = function(key, value) {
|
||||
if (isCallable($replacer) && (value = $replacer.call(this, key, value)), !isSymbol(value)) return value;
|
||||
}), args[1] = replacer, $stringify.apply(null, args);
|
||||
}
|
||||
});
|
||||
}
|
||||
if (!$Symbol[PROTOTYPE][TO_PRIMITIVE]) {
|
||||
var valueOf = $Symbol[PROTOTYPE].valueOf;
|
||||
redefine($Symbol[PROTOTYPE], TO_PRIMITIVE, function() {
|
||||
return valueOf.apply(this, arguments);
|
||||
@ -8112,25 +8123,25 @@
|
||||
},
|
||||
17945: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
"use strict";
|
||||
var ArrayBufferViewCore = __webpack_require__(4351), toLength = __webpack_require__(31998), toOffset = __webpack_require__(11729), toObject = __webpack_require__(89343), fails = __webpack_require__(60232), aTypedArray = ArrayBufferViewCore.aTypedArray;
|
||||
(0, ArrayBufferViewCore.exportTypedArrayMethod)("set", function(arrayLike) {
|
||||
var ArrayBufferViewCore = __webpack_require__(4351), toLength = __webpack_require__(31998), toOffset = __webpack_require__(11729), toObject = __webpack_require__(89343), fails = __webpack_require__(60232), aTypedArray = ArrayBufferViewCore.aTypedArray, exportTypedArrayMethod = ArrayBufferViewCore.exportTypedArrayMethod, FORCED = fails(function() {
|
||||
new Int8Array(1).set({});
|
||||
});
|
||||
exportTypedArrayMethod("set", function(arrayLike) {
|
||||
aTypedArray(this);
|
||||
var offset = toOffset(arguments.length > 1 ? arguments[1] : void 0, 1), length = this.length, src = toObject(arrayLike), len = toLength(src.length), index = 0;
|
||||
if (len + offset > length) throw RangeError("Wrong length");
|
||||
for(; index < len;)this[offset + index] = src[index++];
|
||||
}, fails(function() {
|
||||
new Int8Array(1).set({});
|
||||
}));
|
||||
}, FORCED);
|
||||
},
|
||||
1987: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
"use strict";
|
||||
var ArrayBufferViewCore = __webpack_require__(4351), typedArraySpeciesConstructor = __webpack_require__(50554), fails = __webpack_require__(60232), aTypedArray = ArrayBufferViewCore.aTypedArray, exportTypedArrayMethod = ArrayBufferViewCore.exportTypedArrayMethod, $slice = [].slice;
|
||||
var ArrayBufferViewCore = __webpack_require__(4351), typedArraySpeciesConstructor = __webpack_require__(50554), fails = __webpack_require__(60232), aTypedArray = ArrayBufferViewCore.aTypedArray, exportTypedArrayMethod = ArrayBufferViewCore.exportTypedArrayMethod, $slice = [].slice, FORCED = fails(function() {
|
||||
new Int8Array(1).slice();
|
||||
});
|
||||
exportTypedArrayMethod("slice", function(start, end) {
|
||||
for(var list = $slice.call(aTypedArray(this), start, end), C = typedArraySpeciesConstructor(this), index = 0, length = list.length, result = new C(length); length > index;)result[index] = list[index++];
|
||||
return result;
|
||||
}, fails(function() {
|
||||
new Int8Array(1).slice();
|
||||
}));
|
||||
}, FORCED);
|
||||
},
|
||||
69691: function(__unused_webpack_module, __unused_webpack_exports, __webpack_require__) {
|
||||
"use strict";
|
||||
@ -8723,7 +8734,7 @@
|
||||
pathSize && ("file" != url.scheme || 1 != pathSize || !isWindowsDriveLetter(path[0], !0)) && path.pop();
|
||||
}, SCHEME_START = {}, SCHEME = {}, NO_SCHEME = {}, SPECIAL_RELATIVE_OR_AUTHORITY = {}, PATH_OR_AUTHORITY = {}, RELATIVE = {}, RELATIVE_SLASH = {}, SPECIAL_AUTHORITY_SLASHES = {}, SPECIAL_AUTHORITY_IGNORE_SLASHES = {}, AUTHORITY = {}, HOST = {}, HOSTNAME = {}, PORT = {}, FILE = {}, FILE_SLASH = {}, FILE_HOST = {}, PATH_START = {}, PATH = {}, CANNOT_BE_A_BASE_URL_PATH = {}, QUERY = {}, FRAGMENT = {}, parseURL = function(url, input, stateOverride, base) {
|
||||
var codePoints, chr, bufferCodePoints, failure, state = stateOverride || SCHEME_START, pointer = 0, buffer = "", seenAt = !1, seenBracket = !1, seenPasswordToken = !1;
|
||||
for(stateOverride || (url.scheme = "", url.username = "", url.password = "", url.host = null, url.port = null, url.path = [], url.query = null, url.fragment = null, url.cannotBeABaseURL = !1, input = input.replace(LEADING_AND_TRAILING_C0_CONTROL_OR_SPACE, "")), codePoints = arrayFrom(input = input.replace(TAB_AND_NEW_LINE, "")); pointer <= codePoints.length;){
|
||||
for(stateOverride || (url.scheme = "", url.username = "", url.password = "", url.host = null, url.port = null, url.path = [], url.query = null, url.fragment = null, url.cannotBeABaseURL = !1, input = input.replace(LEADING_AND_TRAILING_C0_CONTROL_OR_SPACE, "")), input = input.replace(TAB_AND_NEW_LINE, ""), codePoints = arrayFrom(input); pointer <= codePoints.length;){
|
||||
switch(chr = codePoints[pointer], state){
|
||||
case SCHEME_START:
|
||||
if (chr && ALPHA.test(chr)) buffer += chr.toLowerCase(), state = SCHEME;
|
||||
@ -8974,13 +8985,14 @@
|
||||
};
|
||||
if (DESCRIPTORS && defineProperties(URLPrototype, {
|
||||
href: accessorDescriptor(serializeURL, function(href) {
|
||||
var url = getInternalURLState(this), failure = parseURL(url, $toString(href));
|
||||
var url = getInternalURLState(this), urlString = $toString(href), failure = parseURL(url, urlString);
|
||||
if (failure) throw TypeError(failure);
|
||||
getInternalSearchParamsState(url.searchParams).updateSearchParams(url.query);
|
||||
}),
|
||||
origin: accessorDescriptor(getOrigin),
|
||||
protocol: accessorDescriptor(getProtocol, function(protocol) {
|
||||
parseURL(getInternalURLState(this), $toString(protocol) + ":", SCHEME_START);
|
||||
var url = getInternalURLState(this);
|
||||
parseURL(url, $toString(protocol) + ":", SCHEME_START);
|
||||
}),
|
||||
username: accessorDescriptor(getUsername, function(username) {
|
||||
var url = getInternalURLState(this), codePoints = arrayFrom($toString(username));
|
||||
@ -10176,7 +10188,8 @@
|
||||
return attachKeys(path, keys);
|
||||
}(path7, keys2) : isarray(path7) ? function(path, keys, options) {
|
||||
for(var parts = [], i = 0; i < path.length; i++)parts.push(pathToRegexp(path[i], keys, options).source);
|
||||
return attachKeys(new RegExp("(?:" + parts.join("|") + ")", flags(options)), keys);
|
||||
var regexp = new RegExp("(?:" + parts.join("|") + ")", flags(options));
|
||||
return attachKeys(regexp, keys);
|
||||
}(path7, keys2, options2) : (path6 = path7, keys1 = keys2, tokensToRegExp(parse(path6, options1 = options2), keys1, options1));
|
||||
}
|
||||
},
|
||||
@ -10415,12 +10428,12 @@
|
||||
}
|
||||
exports.extract = extract, exports.parse = parse, exports.stringify = (object, options4)=>{
|
||||
if (!object) return "";
|
||||
validateArrayFormatSeparator((options4 = Object.assign({
|
||||
options4 = Object.assign({
|
||||
encode: !0,
|
||||
strict: !0,
|
||||
arrayFormat: "none",
|
||||
arrayFormatSeparator: ","
|
||||
}, options4)).arrayFormatSeparator);
|
||||
}, options4), validateArrayFormatSeparator(options4.arrayFormatSeparator);
|
||||
const shouldFilter = (key)=>options4.skipNull && isNullOrUndefined(object[key]) || options4.skipEmptyString && "" === object[key]
|
||||
, formatter = function(options) {
|
||||
switch(options.arrayFormat){
|
||||
@ -11678,7 +11691,7 @@
|
||||
0 !== k ? (d = Rc(k), e = F) : 0 != (h &= f) && (d = Rc(h), e = F);
|
||||
} else 0 != (f = c & ~g) ? (d = Rc(f), e = F) : 0 !== h && (d = Rc(h), e = F);
|
||||
if (0 === d) return 0;
|
||||
if (d = c & ((0 > (d = 31 - Vc(d)) ? 0 : 1 << d) << 1) - 1, 0 !== b && b !== d && 0 == (b & g)) {
|
||||
if (d = 31 - Vc(d), d = c & ((0 > d ? 0 : 1 << d) << 1) - 1, 0 !== b && b !== d && 0 == (b & g)) {
|
||||
if (Rc(b), e <= F) return b;
|
||||
F = e;
|
||||
}
|
||||
@ -11858,21 +11871,21 @@
|
||||
movementY: function(a) {
|
||||
return "movementY" in a ? a.movementY : xd;
|
||||
}
|
||||
}), Bd = rd(Ad), Dd = rd(m({}, Ad, {
|
||||
}), Bd = rd(Ad), Cd = m({}, Ad, {
|
||||
dataTransfer: 0
|
||||
})), Fd = rd(m({}, ud, {
|
||||
}), Dd = rd(Cd), Ed = m({}, ud, {
|
||||
relatedTarget: 0
|
||||
})), Hd = rd(m({}, sd, {
|
||||
}), Fd = rd(Ed), Gd = m({}, sd, {
|
||||
animationName: 0,
|
||||
elapsedTime: 0,
|
||||
pseudoElement: 0
|
||||
})), Jd = rd(m({}, sd, {
|
||||
}), Hd = rd(Gd), Id = m({}, sd, {
|
||||
clipboardData: function(a) {
|
||||
return "clipboardData" in a ? a.clipboardData : window.clipboardData;
|
||||
}
|
||||
})), Ld = rd(m({}, sd, {
|
||||
}), Jd = rd(Id), Kd = m({}, sd, {
|
||||
data: 0
|
||||
})), Md = {
|
||||
}), Ld = rd(Kd), Md = {
|
||||
Esc: "Escape",
|
||||
Spacebar: " ",
|
||||
Left: "ArrowLeft",
|
||||
@ -11935,7 +11948,7 @@
|
||||
function zd() {
|
||||
return Pd;
|
||||
}
|
||||
var Rd = rd(m({}, ud, {
|
||||
var Qd = m({}, ud, {
|
||||
key: function(a) {
|
||||
if (a.key) {
|
||||
var b = Md[a.key] || a.key;
|
||||
@ -11961,7 +11974,7 @@
|
||||
which: function(a) {
|
||||
return "keypress" === a.type ? od(a) : "keydown" === a.type || "keyup" === a.type ? a.keyCode : 0;
|
||||
}
|
||||
})), Td = rd(m({}, Ad, {
|
||||
}), Rd = rd(Qd), Sd = m({}, Ad, {
|
||||
pointerId: 0,
|
||||
width: 0,
|
||||
height: 0,
|
||||
@ -11972,7 +11985,7 @@
|
||||
twist: 0,
|
||||
pointerType: 0,
|
||||
isPrimary: 0
|
||||
})), Vd = rd(m({}, ud, {
|
||||
}), Td = rd(Sd), Ud = m({}, ud, {
|
||||
touches: 0,
|
||||
targetTouches: 0,
|
||||
changedTouches: 0,
|
||||
@ -11981,11 +11994,11 @@
|
||||
ctrlKey: 0,
|
||||
shiftKey: 0,
|
||||
getModifierState: zd
|
||||
})), Xd = rd(m({}, sd, {
|
||||
}), Vd = rd(Ud), Wd = m({}, sd, {
|
||||
propertyName: 0,
|
||||
elapsedTime: 0,
|
||||
pseudoElement: 0
|
||||
})), Zd = rd(m({}, Ad, {
|
||||
}), Xd = rd(Wd), Yd = m({}, Ad, {
|
||||
deltaX: function(a) {
|
||||
return "deltaX" in a ? a.deltaX : "wheelDeltaX" in a ? -a.wheelDeltaX : 0;
|
||||
},
|
||||
@ -11994,7 +12007,7 @@
|
||||
},
|
||||
deltaZ: 0,
|
||||
deltaMode: 0
|
||||
})), $d = [
|
||||
}), Zd = rd(Yd), $d = [
|
||||
9,
|
||||
13,
|
||||
27,
|
||||
@ -12051,7 +12064,8 @@
|
||||
se(a, 0);
|
||||
}
|
||||
function te(a) {
|
||||
if (Wa(ue(a))) return a;
|
||||
var b = ue(a);
|
||||
if (Wa(b)) return a;
|
||||
}
|
||||
function ve(a, b) {
|
||||
if ("change" === a) return b;
|
||||
@ -12726,10 +12740,10 @@
|
||||
}
|
||||
}
|
||||
function gg(a, b) {
|
||||
return Nf(a = fg(a), b);
|
||||
return a = fg(a), Nf(a, b);
|
||||
}
|
||||
function hg(a, b, c) {
|
||||
return Of(a = fg(a), b, c);
|
||||
return a = fg(a), Of(a, b, c);
|
||||
}
|
||||
function ig() {
|
||||
if (null !== bg) {
|
||||
@ -13438,7 +13452,7 @@
|
||||
p.getSnapshot = c7, p.setSnapshot = l;
|
||||
var a = f(b._source);
|
||||
if (!He(g, a)) {
|
||||
He(n, a = c7(b._source)) || (l(a), a = Ig(w), e.mutableReadLanes |= a & e.pendingLanes), a = e.mutableReadLanes, e.entangledLanes |= a;
|
||||
a = c7(b._source), He(n, a) || (l(a), a = Ig(w), e.mutableReadLanes |= a & e.pendingLanes), a = e.mutableReadLanes, e.entangledLanes |= a;
|
||||
for(var d = e.entanglements, h = a; 0 < h;){
|
||||
var k = 31 - Vc(h), v = 1 << k;
|
||||
d[k] |= a, h &= ~v;
|
||||
@ -13472,7 +13486,8 @@
|
||||
}).dispatch = l = Oh.bind(null, R, a21), k3.queue = a21, k3.baseQueue = null, n = Mh(e, b, c7), k3.memoizedState = k3.baseState = n), n;
|
||||
}
|
||||
function Ph(a, b, c) {
|
||||
return Nh(Ih(), a, b, c);
|
||||
var d = Ih();
|
||||
return Nh(d, a, b, c);
|
||||
}
|
||||
function Qh(a) {
|
||||
var b = Hh();
|
||||
@ -13839,13 +13854,13 @@
|
||||
var g = b.stateNode, h = b.memoizedProps;
|
||||
g.props = h;
|
||||
var k = g.context, l = c.contextType;
|
||||
l = "object" == typeof l && null !== l ? vg(l) : Ef(b, l = Ff(c) ? Df : M.current);
|
||||
"object" == typeof l && null !== l ? l = vg(l) : (l = Ff(c) ? Df : M.current, l = Ef(b, l));
|
||||
var n = c.getDerivedStateFromProps, A = "function" == typeof n || "function" == typeof g.getSnapshotBeforeUpdate;
|
||||
A || "function" != typeof g.UNSAFE_componentWillReceiveProps && "function" != typeof g.componentWillReceiveProps || (h !== d || k !== l) && Ng(b, g, d, l), wg = !1;
|
||||
var p = b.memoizedState;
|
||||
g.state = p, Cg(b, d, g, e), k = b.memoizedState, h !== d || p !== k || N.current || wg ? ("function" == typeof n && (Gg(b, c, n, d), k = b.memoizedState), (h = wg || Lg(b, c, h, d, p, k, l)) ? (A || "function" != typeof g.UNSAFE_componentWillMount && "function" != typeof g.componentWillMount || ("function" == typeof g.componentWillMount && g.componentWillMount(), "function" == typeof g.UNSAFE_componentWillMount && g.UNSAFE_componentWillMount()), "function" == typeof g.componentDidMount && (b.flags |= 4)) : ("function" == typeof g.componentDidMount && (b.flags |= 4), b.memoizedProps = d, b.memoizedState = k), g.props = d, g.state = k, g.context = l, d = h) : ("function" == typeof g.componentDidMount && (b.flags |= 4), d = !1);
|
||||
} else {
|
||||
g = b.stateNode, yg(a, b), h = b.memoizedProps, l = b.type === b.elementType ? h : lg(b.type, h), g.props = l, A = b.pendingProps, p = g.context, k = c.contextType, k = "object" == typeof k && null !== k ? vg(k) : Ef(b, k = Ff(c) ? Df : M.current);
|
||||
g = b.stateNode, yg(a, b), h = b.memoizedProps, l = b.type === b.elementType ? h : lg(b.type, h), g.props = l, A = b.pendingProps, p = g.context, k = c.contextType, "object" == typeof k && null !== k ? k = vg(k) : (k = Ff(c) ? Df : M.current, k = Ef(b, k));
|
||||
var C = c.getDerivedStateFromProps;
|
||||
(n = "function" == typeof C || "function" == typeof g.getSnapshotBeforeUpdate) || "function" != typeof g.UNSAFE_componentWillReceiveProps && "function" != typeof g.componentWillReceiveProps || (h !== A || p !== k) && Ng(b, g, d, k), wg = !1, p = b.memoizedState, g.state = p, Cg(b, d, g, e);
|
||||
var x = b.memoizedState;
|
||||
@ -14746,7 +14761,7 @@
|
||||
}
|
||||
15 === b ? (c = Lj.bind(null, a25), null === ag ? (ag = [
|
||||
c
|
||||
], bg = Of(Uf, jg)) : ag.push(c), c = Zf) : c = 14 === b ? hg(99, Lj.bind(null, a25)) : hg(c = function(a) {
|
||||
], bg = Of(Uf, jg)) : ag.push(c), c = Zf) : 14 === b ? c = hg(99, Lj.bind(null, a25)) : (c = function(a) {
|
||||
switch(a){
|
||||
case 15:
|
||||
case 14:
|
||||
@ -14772,7 +14787,7 @@
|
||||
default:
|
||||
throw Error(y(358, a));
|
||||
}
|
||||
}(b), Nj.bind(null, a25)), a25.callbackPriority = b, a25.callbackNode = c;
|
||||
}(b), c = hg(c, Nj.bind(null, a25))), a25.callbackPriority = b, a25.callbackNode = c;
|
||||
}
|
||||
}
|
||||
function Nj(a) {
|
||||
@ -15071,7 +15086,7 @@
|
||||
e[k] = 0, g[k] = -1, h[k] = -1, f &= ~l;
|
||||
}
|
||||
if (null !== Cj && 0 == (24 & d) && Cj.has(a) && Cj.delete(a), a === U && (Y = U = null, W = 0), 1 < c.flags ? null !== c.lastEffect ? (c.lastEffect.nextEffect = c, d = c.firstEffect) : d = c : d = c.firstEffect, null !== d) {
|
||||
if (e = X, X |= 32, pj.current = null, kf = fd, Oe(g = Ne())) {
|
||||
if (e = X, X |= 32, pj.current = null, kf = fd, g = Ne(), Oe(g)) {
|
||||
if ("selectionStart" in g) h = {
|
||||
start: g.selectionStart,
|
||||
end: g.selectionEnd
|
||||
@ -15249,7 +15264,7 @@
|
||||
return X = b, ig(), !0;
|
||||
}
|
||||
function gk(a, b, c) {
|
||||
b = Pi(a, b = Mi(c, b), 1), Ag(a, b), b = Hg(), a = Kj(a, 1), null !== a && ($c(a, 1, b), Mj(a, b));
|
||||
b = Mi(c, b), b = Pi(a, b, 1), Ag(a, b), b = Hg(), null !== (a = Kj(a, 1)) && ($c(a, 1, b), Mj(a, b));
|
||||
}
|
||||
function Wi(a, b) {
|
||||
if (3 === a.tag) gk(a, a, b);
|
||||
@ -15261,7 +15276,8 @@
|
||||
if (1 === c.tag) {
|
||||
var d = c.stateNode;
|
||||
if ("function" == typeof c.type.getDerivedStateFromError || "function" == typeof d.componentDidCatch && (null === Ti || !Ti.has(d))) {
|
||||
var e = Si(c, a = Mi(b, a), 1);
|
||||
a = Mi(b, a);
|
||||
var e = Si(c, a, 1);
|
||||
if (Ag(c, e), e = Hg(), null !== (c = Kj(c, 1))) $c(c, 1, e), Mj(c, e);
|
||||
else if ("function" == typeof d.componentDidCatch && (null === Ti || !Ti.has(d))) try {
|
||||
d.componentDidCatch(b, a);
|
||||
@ -15649,9 +15665,15 @@
|
||||
b[ff] = null;
|
||||
});
|
||||
}, ec = function(a) {
|
||||
13 === a.tag && (Jg(a, 4, Hg()), ok(a, 4));
|
||||
if (13 === a.tag) {
|
||||
var b = Hg();
|
||||
Jg(a, 4, b), ok(a, 4);
|
||||
}
|
||||
}, fc = function(a) {
|
||||
13 === a.tag && (Jg(a, 67108864, Hg()), ok(a, 67108864));
|
||||
if (13 === a.tag) {
|
||||
var b = Hg();
|
||||
Jg(a, 67108864, b), ok(a, 67108864);
|
||||
}
|
||||
}, gc = function(a) {
|
||||
if (13 === a.tag) {
|
||||
var b = Hg(), c = Ig(a);
|
||||
@ -15966,8 +15988,8 @@
|
||||
]);
|
||||
return React.createElement(reactRouter.__RouterContext.Consumer, null, function(r) {
|
||||
r || invariant(!1);
|
||||
var o = r.history, e12 = normalizeToLocation(resolveToLocation(u, r.location), r.location), n = _extends({}, s, {
|
||||
href: e12 ? o.createHref(e12) : "",
|
||||
var o = r.history, e12 = normalizeToLocation(resolveToLocation(u, r.location), r.location), t4 = e12 ? o.createHref(e12) : "", n = _extends({}, s, {
|
||||
href: t4,
|
||||
navigate: function() {
|
||||
var e = resolveToLocation(u, r.location), t = history.createPath(r.location) === history.createPath(normalizeToLocation(e));
|
||||
(c || t ? o.replace : o.push)(e);
|
||||
@ -15980,7 +16002,7 @@
|
||||
}, forwardRef$1 = React.forwardRef;
|
||||
void 0 === forwardRef$1 && (forwardRef$1 = forwardRefShim$1);
|
||||
var NavLink = forwardRef$1(function(e13, s) {
|
||||
var t4 = e13["aria-current"], l = void 0 === t4 ? "page" : t4, r1 = e13.activeClassName, p = void 0 === r1 ? "active" : r1, R = e13.activeStyle, h = e13.className, y = e13.exact, d = e13.isActive, m = e13.location, v = e13.sensitive, b = e13.strict, P = e13.style, w = e13.to, x = e13.innerRef, g = _objectWithoutPropertiesLoose(e13, [
|
||||
var t5 = e13["aria-current"], l = void 0 === t5 ? "page" : t5, r1 = e13.activeClassName, p = void 0 === r1 ? "active" : r1, R = e13.activeStyle, h = e13.className, y = e13.exact, d = e13.isActive, m = e13.location, v = e13.sensitive, b = e13.strict, P = e13.style, w = e13.to, x = e13.innerRef, g = _objectWithoutPropertiesLoose(e13, [
|
||||
"aria-current",
|
||||
"activeClassName",
|
||||
"activeStyle",
|
||||
@ -15996,12 +16018,12 @@
|
||||
]);
|
||||
return React.createElement(reactRouter.__RouterContext.Consumer, null, function(e14) {
|
||||
e14 || invariant(!1);
|
||||
var t5 = m || e14.location, r2 = normalizeToLocation(resolveToLocation(w, t5), t5), o = r2.pathname, n = o && o.replace(/([.+*?=^!:${}()[\]|/\\])/g, "\\$1"), a = n ? reactRouter.matchPath(t5.pathname, {
|
||||
var t6 = m || e14.location, r2 = normalizeToLocation(resolveToLocation(w, t6), t6), o = r2.pathname, n = o && o.replace(/([.+*?=^!:${}()[\]|/\\])/g, "\\$1"), a = n ? reactRouter.matchPath(t6.pathname, {
|
||||
path: n,
|
||||
exact: y,
|
||||
sensitive: v,
|
||||
strict: b
|
||||
}) : null, i = !!(d ? d(a, t5) : a), c = "function" == typeof h ? h(i) : h, u = "function" == typeof P ? P(i) : P;
|
||||
}) : null, i = !!(d ? d(a, t6) : a), c = "function" == typeof h ? h(i) : h, u = "function" == typeof P ? P(i) : P;
|
||||
i && (c = function() {
|
||||
for(var e15 = arguments.length, t = new Array(e15), r = 0; r < e15; r++)t[r] = arguments[r];
|
||||
return t.filter(function(e) {
|
||||
|
@ -1,7 +1,7 @@
|
||||
export default ((adler, buf, len, pos)=>{
|
||||
let s1 = 0xffff & adler | 0, s2 = adler >>> 16 & 0xffff | 0, n = 0;
|
||||
for(; 0 !== len;){
|
||||
len -= n = len > 2000 ? 2000 : len;
|
||||
n = len > 2000 ? 2000 : len, len -= n;
|
||||
do s2 = s2 + (s1 = s1 + buf[pos++] | 0) | 0;
|
||||
while (--n)
|
||||
s1 %= 65521, s2 %= 65521;
|
||||
|
@ -632,10 +632,10 @@
|
||||
}(function(rule) {
|
||||
currentSheet.insert(rule);
|
||||
}),
|
||||
], serializer = (length = Utility_sizeof(collection = [
|
||||
], serializer = (collection = [
|
||||
compat,
|
||||
removeLabel
|
||||
].concat(stylisPlugins, finalizingPlugins)), function(element, index, children, callback) {
|
||||
].concat(stylisPlugins, finalizingPlugins), length = Utility_sizeof(collection), function(element, index, children, callback) {
|
||||
for(var output = "", i = 0; i < length; i++)output += collection[i](element, index, children, callback) || "";
|
||||
return output;
|
||||
}), stylis = function(styles) {
|
||||
@ -679,7 +679,8 @@
|
||||
}
|
||||
}, Global = function(func) {
|
||||
return (0, react.forwardRef)(function(props, ref) {
|
||||
return func(props, (0, react.useContext)(EmotionCacheContext), ref);
|
||||
var cache = (0, react.useContext)(EmotionCacheContext);
|
||||
return func(props, cache, ref);
|
||||
});
|
||||
}(function(props, cache) {
|
||||
var serialized = emotion_serialize_browser_esm_serializeStyles([
|
||||
|
@ -1095,7 +1095,7 @@
|
||||
}
|
||||
return b;
|
||||
}, k.set = function(a, b) {
|
||||
return V(this), this.i = null, ed(this, a = W(this, a)) && (this.h -= this.g.get(a).length), this.g.set(a, [
|
||||
return V(this), this.i = null, a = W(this, a), ed(this, a) && (this.h -= this.g.get(a).length), this.g.set(a, [
|
||||
b
|
||||
]), this.h += 1, this;
|
||||
}, k.get = function(a, b) {
|
||||
@ -1466,7 +1466,7 @@
|
||||
if (1 == d) {
|
||||
c = b.s ? b.s.length : 0, b = Date.now() - b.F;
|
||||
var a8, b7, e = a.C;
|
||||
D(d = Sb(), new Vb(d, c, b, e)), Hc(a);
|
||||
d = Sb(), D(d, new Vb(d, c, b, e)), Hc(a);
|
||||
} else Gc(a);
|
||||
} else if (3 == (e = b.o) || 0 == e && 0 < a.I || !(1 == d && (a8 = a, b7 = b, !(Cc(a8.i) >= a8.i.j - (a8.m ? 1 : 0)) && (a8.m ? (a8.l = b7.D.concat(a8.l), !0) : 1 != a8.G && 2 != a8.G && !(a8.C >= (a8.Xa ? 0 : a8.Ya)) && (a8.m = K(q(a8.Ha, a8, b7), Od(a8, a8.C)), a8.C++, !0))) || 2 == d && Bc(a))) switch(c && 0 < c.length && ((b = a.i).i = b.i.concat(c)), e){
|
||||
case 1:
|
||||
@ -1680,7 +1680,7 @@
|
||||
b = 1e3;
|
||||
}
|
||||
else b = 1e3;
|
||||
b = Pd(this, e, b), R(c = N(this.F), "RID", a), R(c, "CVER", 22), this.D && R(c, "X-HTTP-Session-Id", this.D), Kd(this, c), this.o && f && Gd(c, this.o, f), Dc(this.i, e), this.Ra && R(c, "TYPE", "init"), this.ja ? (R(c, "$req", b), R(c, "SID", "null"), e.$ = !0, ic(e, c, null)) : ic(e, c, b), this.G = 2;
|
||||
b = Pd(this, e, b), c = N(this.F), R(c, "RID", a), R(c, "CVER", 22), this.D && R(c, "X-HTTP-Session-Id", this.D), Kd(this, c), this.o && f && Gd(c, this.o, f), Dc(this.i, e), this.Ra && R(c, "TYPE", "init"), this.ja ? (R(c, "$req", b), R(c, "SID", "null"), e.$ = !0, ic(e, c, null)) : ic(e, c, b), this.G = 2;
|
||||
}
|
||||
} else 3 == this.G && (a ? Qd(this, a) : 0 == this.l.length || id(this.i) || Qd(this));
|
||||
}
|
||||
|
@ -5,7 +5,7 @@ export function treeSubTree(tree, pathObj) {
|
||||
children: {},
|
||||
childCount: 0
|
||||
};
|
||||
child = new Tree(next, child, childNode), next = pathGetFront(path = pathPopFront(path));
|
||||
child = new Tree(next, child, childNode), path = pathPopFront(path), next = pathGetFront(path);
|
||||
}
|
||||
return child;
|
||||
}
|
||||
|
@ -980,8 +980,8 @@
|
||||
}
|
||||
function createAdder(direction, name) {
|
||||
return function(val, period) {
|
||||
var tmp;
|
||||
return null === period || isNaN(+period) || (deprecateSimple(name, "moment()." + name + "(period, number) is deprecated. Please use moment()." + name + "(number, period). See http://momentjs.com/guides/#/warnings/add-inverted-param/ for more info."), tmp = val, val = period, period = tmp), addSubtract(this, createDuration(val, period), direction), this;
|
||||
var dur, tmp;
|
||||
return null === period || isNaN(+period) || (deprecateSimple(name, "moment()." + name + "(period, number) is deprecated. Please use moment()." + name + "(number, period). See http://momentjs.com/guides/#/warnings/add-inverted-param/ for more info."), tmp = val, val = period, period = tmp), dur = createDuration(val, period), addSubtract(this, dur, direction), this;
|
||||
};
|
||||
}
|
||||
function addSubtract(mom, duration, isAdding, updateOffset) {
|
||||
@ -1036,7 +1036,7 @@
|
||||
}
|
||||
function getSetWeekYearHelper(input, week, weekday, dow, doy) {
|
||||
var weeksTarget;
|
||||
return null == input ? weekOfYear(this, dow, doy).year : (week > (weeksTarget = weeksInYear(input, dow, doy)) && (week = weeksTarget), setWeekAll.call(this, input, week, weekday, dow, doy));
|
||||
return null == input ? weekOfYear(this, dow, doy).year : (weeksTarget = weeksInYear(input, dow, doy), week > weeksTarget && (week = weeksTarget), setWeekAll.call(this, input, week, weekday, dow, doy));
|
||||
}
|
||||
function setWeekAll(weekYear, week, weekday, dow, doy) {
|
||||
var dayOfYearData = dayOfYearFromWeeks(weekYear, week, weekday, dow, doy), date = createUTCDate(dayOfYearData.year, 0, dayOfYearData.dayOfYear);
|
||||
@ -1799,7 +1799,7 @@
|
||||
return this.isValid() ? this._milliseconds + 864e5 * this._days + this._months % 12 * 2592e6 + 31536e6 * toInt(this._months / 12) : NaN;
|
||||
}, proto$2._bubble = function() {
|
||||
var seconds, minutes, hours, years, monthsFromDays, milliseconds = this._milliseconds, days = this._days, months = this._months, data = this._data;
|
||||
return milliseconds >= 0 && days >= 0 && months >= 0 || milliseconds <= 0 && days <= 0 && months <= 0 || (milliseconds += 864e5 * absCeil(monthsToDays(months) + days), days = 0, months = 0), data.milliseconds = milliseconds % 1000, seconds = absFloor(milliseconds / 1000), data.seconds = seconds % 60, minutes = absFloor(seconds / 60), data.minutes = minutes % 60, hours = absFloor(minutes / 60), data.hours = hours % 24, days += absFloor(hours / 24), months += monthsFromDays = absFloor(daysToMonths(days)), days -= absCeil(monthsToDays(monthsFromDays)), years = absFloor(months / 12), months %= 12, data.days = days, data.months = months, data.years = years, this;
|
||||
return milliseconds >= 0 && days >= 0 && months >= 0 || milliseconds <= 0 && days <= 0 && months <= 0 || (milliseconds += 864e5 * absCeil(monthsToDays(months) + days), days = 0, months = 0), data.milliseconds = milliseconds % 1000, seconds = absFloor(milliseconds / 1000), data.seconds = seconds % 60, minutes = absFloor(seconds / 60), data.minutes = minutes % 60, hours = absFloor(minutes / 60), data.hours = hours % 24, days += absFloor(hours / 24), monthsFromDays = absFloor(daysToMonths(days)), months += monthsFromDays, days -= absCeil(monthsToDays(monthsFromDays)), years = absFloor(months / 12), months %= 12, data.days = days, data.months = months, data.years = years, this;
|
||||
}, proto$2.clone = function() {
|
||||
return createDuration(this);
|
||||
}, proto$2.get = function(units) {
|
||||
@ -1809,7 +1809,7 @@
|
||||
}, proto$2.months = months1, proto$2.years = years1, proto$2.humanize = function(argWithSuffix, argThresholds) {
|
||||
if (!this.isValid()) return this.localeData().invalidDate();
|
||||
var locale, output, posNegDuration, withoutSuffix, thresholds1, locale3, duration, seconds, minutes, hours, days, months, weeks, years, a, withSuffix = !1, th = thresholds;
|
||||
return "object" == typeof argWithSuffix && (argThresholds = argWithSuffix, argWithSuffix = !1), "boolean" == typeof argWithSuffix && (withSuffix = argWithSuffix), "object" == typeof argThresholds && (th = Object.assign({}, thresholds, argThresholds), null != argThresholds.s && null == argThresholds.ss && (th.ss = argThresholds.s - 1)), locale = this.localeData(), output = (posNegDuration = this, withoutSuffix = !withSuffix, thresholds1 = th, locale3 = locale, seconds = round((duration = createDuration(posNegDuration).abs()).as("s")), minutes = round(duration.as("m")), hours = round(duration.as("h")), days = round(duration.as("d")), months = round(duration.as("M")), weeks = round(duration.as("w")), years = round(duration.as("y")), a = seconds <= thresholds1.ss && [
|
||||
return "object" == typeof argWithSuffix && (argThresholds = argWithSuffix, argWithSuffix = !1), "boolean" == typeof argWithSuffix && (withSuffix = argWithSuffix), "object" == typeof argThresholds && (th = Object.assign({}, thresholds, argThresholds), null != argThresholds.s && null == argThresholds.ss && (th.ss = argThresholds.s - 1)), locale = this.localeData(), output = (posNegDuration = this, withoutSuffix = !withSuffix, thresholds1 = th, locale3 = locale, duration = createDuration(posNegDuration).abs(), seconds = round(duration.as("s")), minutes = round(duration.as("m")), hours = round(duration.as("h")), days = round(duration.as("d")), months = round(duration.as("M")), weeks = round(duration.as("w")), years = round(duration.as("y")), a = seconds <= thresholds1.ss && [
|
||||
"s",
|
||||
seconds
|
||||
] || seconds < thresholds1.s && [
|
||||
|
@ -1210,8 +1210,8 @@
|
||||
function(module, exports) {
|
||||
var objectProto = Object.prototype;
|
||||
module.exports = function(value) {
|
||||
var Ctor = value && value.constructor;
|
||||
return value === ("function" == typeof Ctor && Ctor.prototype || objectProto);
|
||||
var Ctor = value && value.constructor, proto = "function" == typeof Ctor && Ctor.prototype || objectProto;
|
||||
return value === proto;
|
||||
};
|
||||
},
|
||||
function(module2, exports, __webpack_require__) {
|
||||
|
@ -116,9 +116,9 @@ var ItemsList = function(_Component) {
|
||||
if (!(instance instanceof Constructor)) throw new TypeError("Cannot call a class as a function");
|
||||
}(this, ItemsList1);
|
||||
for(var _len = arguments.length, args = new Array(_len), _key = 0; _key < _len; _key++)args[_key] = arguments[_key];
|
||||
return _defineProperty(_assertThisInitialized(_this = _super.call.apply(_super, [
|
||||
return _this = _super.call.apply(_super, [
|
||||
this
|
||||
].concat(args))), "storeHighlightedItemReference", function(highlightedItem) {
|
||||
].concat(args)), _defineProperty(_assertThisInitialized(_this), "storeHighlightedItemReference", function(highlightedItem) {
|
||||
_this.props.onHighlightedItemChange(null === highlightedItem ? null : highlightedItem.item);
|
||||
}), _this;
|
||||
}
|
||||
|
@ -3,6 +3,6 @@ import { useRouter } from "next/router";
|
||||
import { useProject } from "@swr/use-project";
|
||||
import useTeam from "@swr/use-team";
|
||||
export default function MyComp() {
|
||||
var projectInfo = useProject(useRouter().query.project).data;
|
||||
var projectName = useRouter().query.project, projectInfo = useProject(projectName).data;
|
||||
return useTeam().teamSlug, useProjectBranches(null == projectInfo ? void 0 : projectInfo.id).data, _jsx(_Fragment, {});
|
||||
};
|
||||
|
@ -1336,11 +1336,13 @@
|
||||
}
|
||||
firstChild = wrap.firstChild;
|
||||
}
|
||||
return firstChild && 1 == firstChild.nodeType && firstChild.setAttribute("data-pm-slice", openStart + " " + openEnd + " " + JSON.stringify(context)), {
|
||||
firstChild && 1 == firstChild.nodeType && firstChild.setAttribute("data-pm-slice", openStart + " " + openEnd + " " + JSON.stringify(context));
|
||||
var text = view.someProp("clipboardTextSerializer", function(f) {
|
||||
return f(slice);
|
||||
}) || slice.content.textBetween(0, slice.content.size, "\n\n");
|
||||
return {
|
||||
dom: wrap,
|
||||
text: view.someProp("clipboardTextSerializer", function(f) {
|
||||
return f(slice);
|
||||
}) || slice.content.textBetween(0, slice.content.size, "\n\n")
|
||||
text: text
|
||||
};
|
||||
}
|
||||
function parseFromClipboard(view, text, html, plainText, $context) {
|
||||
@ -1613,10 +1615,10 @@
|
||||
var ref = mut.addedNodes[i$1], previousSibling = ref.previousSibling, nextSibling = ref.nextSibling;
|
||||
(!previousSibling || 0 > Array.prototype.indexOf.call(mut.addedNodes, previousSibling)) && (prev = previousSibling), (!nextSibling || 0 > Array.prototype.indexOf.call(mut.addedNodes, nextSibling)) && (next = nextSibling);
|
||||
}
|
||||
var fromOffset = prev && prev.parentNode == mut.target ? domIndex(prev) + 1 : 0, from = desc.localPosFromDOM(mut.target, fromOffset, -1), toOffset = next && next.parentNode == mut.target ? domIndex(next) : mut.target.childNodes.length;
|
||||
var fromOffset = prev && prev.parentNode == mut.target ? domIndex(prev) + 1 : 0, from = desc.localPosFromDOM(mut.target, fromOffset, -1), toOffset = next && next.parentNode == mut.target ? domIndex(next) : mut.target.childNodes.length, to = desc.localPosFromDOM(mut.target, toOffset, 1);
|
||||
return {
|
||||
from: from,
|
||||
to: desc.localPosFromDOM(mut.target, toOffset, 1)
|
||||
to: to
|
||||
};
|
||||
}
|
||||
return "attributes" == mut.type ? {
|
||||
@ -2168,7 +2170,7 @@
|
||||
} else mustRebuild = !0;
|
||||
}
|
||||
if (mustRebuild) {
|
||||
var built = buildTree(mapAndGatherRemainingDecorations(children, oldChildren, newLocal || [], mapping, offset, oldOffset, options), node, 0, options);
|
||||
var decorations = mapAndGatherRemainingDecorations(children, oldChildren, newLocal || [], mapping, offset, oldOffset, options), built = buildTree(decorations, node, 0, options);
|
||||
newLocal = built.local;
|
||||
for(var i$2 = 0; i$2 < children.length; i$2 += 3)children[i$2 + 1] < 0 && (children.splice(i$2, 3), i$2 -= 3);
|
||||
for(var i$3 = 0, j = 0; i$3 < built.children.length; i$3 += 3){
|
||||
@ -2367,7 +2369,14 @@
|
||||
var adjust = Math.max(0, start - Math.min(endA, endB));
|
||||
preferredPos -= endA + adjust - start;
|
||||
}
|
||||
return endA < start && a.size < b.size ? (start -= preferredPos <= start && preferredPos >= endA ? start - preferredPos : 0, endB = start + (endB - endA), endA = start) : endB < start && (start -= preferredPos <= start && preferredPos >= endB ? start - preferredPos : 0, endA = start + (endA - endB), endB = start), {
|
||||
if (endA < start && a.size < b.size) {
|
||||
var move = preferredPos <= start && preferredPos >= endA ? start - preferredPos : 0;
|
||||
start -= move, endB = start + (endB - endA), endA = start;
|
||||
} else if (endB < start) {
|
||||
var move$1 = preferredPos <= start && preferredPos >= endB ? start - preferredPos : 0;
|
||||
start -= move$1, endA = start + (endA - endB), endB = start;
|
||||
}
|
||||
return {
|
||||
start: start,
|
||||
endA: endA,
|
||||
endB: endB
|
||||
|
@ -630,11 +630,11 @@
|
||||
if ("function" != typeof listener) throw new Error("Invalid listener for " + objName(obj) + "#" + fnName + "; must be a function.");
|
||||
}, normalizeListenArgs = function(self, args, fnName) {
|
||||
var target, type, listener, isTargetingSelf = args.length < 3 || args[0] === self || args[0] === self.eventBusEl_;
|
||||
return isTargetingSelf ? (target = self.eventBusEl_, args.length >= 3 && args.shift(), type = args[0], listener = args[1]) : (target = args[0], type = args[1], listener = args[2]), validateTarget(target, self, fnName), validateEventType(type, self, fnName), validateListener(listener, self, fnName), {
|
||||
return isTargetingSelf ? (target = self.eventBusEl_, args.length >= 3 && args.shift(), type = args[0], listener = args[1]) : (target = args[0], type = args[1], listener = args[2]), validateTarget(target, self, fnName), validateEventType(type, self, fnName), validateListener(listener, self, fnName), listener = bind(self, listener), {
|
||||
isTargetingSelf: isTargetingSelf,
|
||||
target: target,
|
||||
type: type,
|
||||
listener: listener = bind(self, listener)
|
||||
listener: listener
|
||||
};
|
||||
}, listen = function(target, method, type, listener) {
|
||||
validateTarget(target, target, method), target.nodeName ? Events[method](target, type, listener) : target[method](type, listener);
|
||||
@ -955,7 +955,7 @@
|
||||
}, _proto.currentDimension = function(widthOrHeight) {
|
||||
var computedWidthOrHeight = 0;
|
||||
if ("width" !== widthOrHeight && "height" !== widthOrHeight) throw new Error("currentDimension only accepts width or height value");
|
||||
if (0 === (computedWidthOrHeight = parseFloat(computedWidthOrHeight = computedStyle(this.el_, widthOrHeight))) || isNaN(computedWidthOrHeight)) {
|
||||
if (computedWidthOrHeight = computedStyle(this.el_, widthOrHeight), 0 === (computedWidthOrHeight = parseFloat(computedWidthOrHeight)) || isNaN(computedWidthOrHeight)) {
|
||||
var rule = "offset" + toTitleCase$1(widthOrHeight);
|
||||
computedWidthOrHeight = this.el_[rule];
|
||||
}
|
||||
@ -2364,12 +2364,12 @@
|
||||
(0, _babel_runtime_helpers_inheritsLoose__WEBPACK_IMPORTED_MODULE_16__.Z)(Button, _ClickableComponent);
|
||||
var _proto = Button.prototype;
|
||||
return _proto.createEl = function(tag, props, attributes) {
|
||||
void 0 === props && (props = {}), void 0 === attributes && (attributes = {});
|
||||
var el = createEl("button", props = assign({
|
||||
void 0 === props && (props = {}), void 0 === attributes && (attributes = {}), tag = "button", props = assign({
|
||||
className: this.buildCSSClass()
|
||||
}, props), attributes = assign({
|
||||
type: "button"
|
||||
}, attributes));
|
||||
}, attributes);
|
||||
var el = createEl(tag, props, attributes);
|
||||
return el.appendChild(createEl("span", {
|
||||
className: "vjs-icon-placeholder"
|
||||
}, {
|
||||
@ -2478,7 +2478,7 @@
|
||||
PlayToggle1.prototype.controlText_ = "Play", Component$1.registerComponent("PlayToggle", PlayToggle1);
|
||||
var defaultImplementation = function(seconds, guide) {
|
||||
var s = Math.floor((seconds = seconds < 0 ? 0 : seconds) % 60), m = Math.floor(seconds / 60 % 60), h = Math.floor(seconds / 3600), gm = Math.floor(guide / 60 % 60), gh = Math.floor(guide / 3600);
|
||||
return (isNaN(seconds) || seconds === 1 / 0) && (h = m = s = "-"), m = (((h = h > 0 || gh > 0 ? h + ":" : "") || gm >= 10) && m < 10 ? "0" + m : m) + ":", h + m + (s = s < 10 ? "0" + s : s);
|
||||
return (isNaN(seconds) || seconds === 1 / 0) && (h = m = s = "-"), m = (((h = h > 0 || gh > 0 ? h + ":" : "") || gm >= 10) && m < 10 ? "0" + m : m) + ":", s = s < 10 ? "0" + s : s, h + m + s;
|
||||
}, implementation = defaultImplementation;
|
||||
function setFormatTime(customImplementation) {
|
||||
implementation = customImplementation;
|
||||
@ -4787,7 +4787,7 @@
|
||||
el.parentNode && el.parentNode.insertBefore(clone, el), Html5.disposeMediaElement(el), el = clone;
|
||||
} else {
|
||||
el = global_document__WEBPACK_IMPORTED_MODULE_1___default().createElement("video");
|
||||
var attributes = mergeOptions$3({}, this.options_.tag && getAttributes(this.options_.tag));
|
||||
var tagAttributes = this.options_.tag && getAttributes(this.options_.tag), attributes = mergeOptions$3({}, tagAttributes);
|
||||
TOUCH_ENABLED && !0 === this.options_.nativeControlsForTouch || delete attributes.controls, setAttributes(el, assign(attributes, {
|
||||
id: this.options_.techId,
|
||||
class: "vjs-tech"
|
||||
@ -5700,7 +5700,7 @@
|
||||
vol = Math.max(0, Math.min(1, parseFloat(percentAsDecimal))), this.cache_.volume = vol, this.techCall_("setVolume", vol), vol > 0 && this.lastVolume_(vol);
|
||||
return;
|
||||
}
|
||||
return isNaN(vol = parseFloat(this.techGet_("volume"))) ? 1 : vol;
|
||||
return vol = parseFloat(this.techGet_("volume")), isNaN(vol) ? 1 : vol;
|
||||
}, _proto.muted = function(_muted) {
|
||||
if (void 0 !== _muted) {
|
||||
this.techCall_("setMuted", _muted);
|
||||
@ -6609,7 +6609,7 @@
|
||||
if (null === expired) return null;
|
||||
expired = expired || 0;
|
||||
var lastSegmentEndTime = intervalDuration(playlist, playlist.mediaSequence + playlist.segments.length, expired);
|
||||
return useSafeLiveEnd && (lastSegmentEndTime -= liveEdgePadding = "number" == typeof liveEdgePadding ? liveEdgePadding : liveEdgeDelay(null, playlist)), Math.max(0, lastSegmentEndTime);
|
||||
return useSafeLiveEnd && (liveEdgePadding = "number" == typeof liveEdgePadding ? liveEdgePadding : liveEdgeDelay(null, playlist), lastSegmentEndTime -= liveEdgePadding), Math.max(0, lastSegmentEndTime);
|
||||
}, isBlacklisted = function(playlist) {
|
||||
return playlist.excludeUntil && playlist.excludeUntil > Date.now();
|
||||
}, isIncompatible = function(playlist) {
|
||||
@ -7192,8 +7192,8 @@
|
||||
var nextSegmentStart = playlist.segments[i + 1].dateTimeObject;
|
||||
if (dateTimeObject < nextSegmentStart) break;
|
||||
}
|
||||
var videoTimingInfo, lastSegment = playlist.segments[playlist.segments.length - 1], lastSegmentStart = lastSegment.dateTimeObject, lastSegmentDuration = lastSegment.videoTimingInfo ? (videoTimingInfo = lastSegment.videoTimingInfo).transmuxedPresentationEnd - videoTimingInfo.transmuxedPresentationStart - videoTimingInfo.transmuxerPrependedSeconds : lastSegment.duration + 0.25 * lastSegment.duration;
|
||||
return dateTimeObject > new Date(lastSegmentStart.getTime() + 1000 * lastSegmentDuration) ? null : (dateTimeObject > lastSegmentStart && (segment = lastSegment), {
|
||||
var videoTimingInfo, lastSegment = playlist.segments[playlist.segments.length - 1], lastSegmentStart = lastSegment.dateTimeObject, lastSegmentDuration = lastSegment.videoTimingInfo ? (videoTimingInfo = lastSegment.videoTimingInfo).transmuxedPresentationEnd - videoTimingInfo.transmuxedPresentationStart - videoTimingInfo.transmuxerPrependedSeconds : lastSegment.duration + 0.25 * lastSegment.duration, lastSegmentEnd = new Date(lastSegmentStart.getTime() + 1000 * lastSegmentDuration);
|
||||
return dateTimeObject > lastSegmentEnd ? null : (dateTimeObject > lastSegmentStart && (segment = lastSegment), {
|
||||
segment: segment,
|
||||
estimatedStart: segment.videoTimingInfo ? segment.videoTimingInfo.transmuxedPresentationStart : Playlist.duration(playlist, playlist.mediaSequence + playlist.segments.indexOf(segment)),
|
||||
type: segment.videoTimingInfo ? "accurate" : "estimate"
|
||||
@ -8477,7 +8477,7 @@
|
||||
},
|
||||
generateSampleTable: function(gops, baseDataOffset) {
|
||||
var h, i, sample, currentGop, dataOffset = baseDataOffset || 0, samples = [];
|
||||
for(h = 0; h < gops.length; h++)for(i = 0, currentGop = gops[h]; i < currentGop.length; i++)dataOffset += (sample = sampleForFrame(currentGop[i], dataOffset)).size, samples.push(sample);
|
||||
for(h = 0; h < gops.length; h++)for(i = 0, currentGop = gops[h]; i < currentGop.length; i++)sample = sampleForFrame(currentGop[i], dataOffset), dataOffset += sample.size, samples.push(sample);
|
||||
return samples;
|
||||
},
|
||||
concatenateNalData: function(gops) {
|
||||
@ -9656,7 +9656,7 @@
|
||||
workingBytes.set(workingData.subarray(position, position + availableBytes)), workingWord = new DataView(workingBytes.buffer).getUint32(0), workingBitsAvailable = 8 * availableBytes, workingBytesAvailable -= availableBytes;
|
||||
}, this.skipBits = function(count) {
|
||||
var skipBytes;
|
||||
workingBitsAvailable > count ? (workingWord <<= count, workingBitsAvailable -= count) : (count -= workingBitsAvailable, count -= 8 * (skipBytes = Math.floor(count / 8)), workingBytesAvailable -= skipBytes, this.loadWord(), workingWord <<= count, workingBitsAvailable -= count);
|
||||
workingBitsAvailable > count ? (workingWord <<= count, workingBitsAvailable -= count) : (count -= workingBitsAvailable, skipBytes = Math.floor(count / 8), count -= 8 * skipBytes, workingBytesAvailable -= skipBytes, this.loadWord(), workingWord <<= count, workingBitsAvailable -= count);
|
||||
}, this.readBits = function(size) {
|
||||
var bits = Math.min(workingBitsAvailable, size), valu = workingWord >>> 32 - bits;
|
||||
return ((workingBitsAvailable -= bits) > 0 ? workingWord <<= bits : workingBytesAvailable > 0 && this.loadWord(), (bits = size - bits) > 0) ? valu << bits | this.readBits(bits) : valu;
|
||||
@ -10291,7 +10291,7 @@
|
||||
}
|
||||
}, parseType_1 = function(buffer) {
|
||||
var result = "";
|
||||
return result += String.fromCharCode(buffer[0]), result += String.fromCharCode(buffer[1]), result += String.fromCharCode(buffer[2]), result += String.fromCharCode(buffer[3]), result;
|
||||
return result += String.fromCharCode(buffer[0]), result += String.fromCharCode(buffer[1]), result += String.fromCharCode(buffer[2]), result += String.fromCharCode(buffer[3]);
|
||||
}, toUnsigned$2 = bin.toUnsigned, findBox_1 = function findBox(data, path) {
|
||||
var i, size, type, end, subresults, results = [];
|
||||
if (!path.length) return null;
|
||||
@ -10386,14 +10386,14 @@
|
||||
traf: matchingTraf
|
||||
});
|
||||
}), mdatTrafPairs.forEach(function(pair) {
|
||||
var result, mdat = pair.mdat, traf = pair.traf, tfhd = findBox_1(traf, [
|
||||
var samples, result, mdat = pair.mdat, traf = pair.traf, tfhd = findBox_1(traf, [
|
||||
"tfhd"
|
||||
]), headerInfo = parseTfhd(tfhd[0]), trackId = headerInfo.trackId, tfdt = findBox_1(traf, [
|
||||
"tfdt"
|
||||
]), baseMediaDecodeTime = tfdt.length > 0 ? parseTfdt(tfdt[0]).baseMediaDecodeTime : 0, truns = findBox_1(traf, [
|
||||
"trun"
|
||||
]);
|
||||
videoTrackId === trackId && truns.length > 0 && (result = findSeiNals(mdat, parseSamples(truns, baseMediaDecodeTime, headerInfo), trackId), captionNals[trackId] || (captionNals[trackId] = {
|
||||
videoTrackId === trackId && truns.length > 0 && (samples = parseSamples(truns, baseMediaDecodeTime, headerInfo), result = findSeiNals(mdat, samples, trackId), captionNals[trackId] || (captionNals[trackId] = {
|
||||
seiNals: [],
|
||||
logs: []
|
||||
}), captionNals[trackId].seiNals = captionNals[trackId].seiNals.concat(result.seiNals), captionNals[trackId].logs = captionNals[trackId].logs.concat(result.logs));
|
||||
@ -11578,7 +11578,7 @@
|
||||
});
|
||||
}, comparePlaylistBandwidth = function(left, right) {
|
||||
var leftBandwidth, rightBandwidth;
|
||||
return left.attributes.BANDWIDTH && (leftBandwidth = left.attributes.BANDWIDTH), leftBandwidth = leftBandwidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE, right.attributes.BANDWIDTH && (rightBandwidth = right.attributes.BANDWIDTH), leftBandwidth - (rightBandwidth = rightBandwidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE);
|
||||
return left.attributes.BANDWIDTH && (leftBandwidth = left.attributes.BANDWIDTH), leftBandwidth = leftBandwidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE, right.attributes.BANDWIDTH && (rightBandwidth = right.attributes.BANDWIDTH), rightBandwidth = rightBandwidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE, leftBandwidth - rightBandwidth;
|
||||
}, simpleSelector = function(master, playerBandwidth, playerWidth, playerHeight, limitRenditionByPlayerDimensions, masterPlaylistController) {
|
||||
if (master) {
|
||||
var resolutionPlusOneList, resolutionPlusOneSmallest, resolutionPlusOneRep, leastPixelDiffRep, options = {
|
||||
@ -13325,15 +13325,15 @@
|
||||
}, _proto.dispose = function() {
|
||||
this.trigger("dispose"), this.pendingTimelineChanges_ = {}, this.lastTimelineChanges_ = {}, this.off();
|
||||
}, TimelineChangeController;
|
||||
}(videojs.EventTarget), Decrypter1 = factory(transform1(getWorkerString(function() {
|
||||
}(videojs.EventTarget), workerCode = transform1(getWorkerString(function() {
|
||||
function createCommonjsModule(fn, basedir, module) {
|
||||
return fn(module = {
|
||||
return module = {
|
||||
path: basedir,
|
||||
exports: {},
|
||||
require: function(path, base) {
|
||||
return commonjsRequire(path, null == base ? module.path : base);
|
||||
}
|
||||
}, module.exports), module.exports;
|
||||
}, fn(module, module.exports), module.exports;
|
||||
}
|
||||
function commonjsRequire() {
|
||||
throw new Error("Dynamic requires are not currently supported by @rollup/plugin-commonjs");
|
||||
@ -13503,7 +13503,7 @@
|
||||
]);
|
||||
});
|
||||
};
|
||||
}))), audioTrackKind_ = function(properties) {
|
||||
})), Decrypter1 = factory(workerCode), audioTrackKind_ = function(properties) {
|
||||
var kind = properties.default ? "main" : "alternative";
|
||||
return properties.characteristics && properties.characteristics.indexOf("public.accessibility.describes-video") >= 0 && (kind = "main-desc"), kind;
|
||||
}, stopLoaders = function(segmentLoader, mediaType) {
|
||||
@ -14699,7 +14699,7 @@
|
||||
comparePlaylistBandwidth: comparePlaylistBandwidth,
|
||||
comparePlaylistResolution: function(left, right) {
|
||||
var leftWidth, rightWidth;
|
||||
return (left.attributes.RESOLUTION && left.attributes.RESOLUTION.width && (leftWidth = left.attributes.RESOLUTION.width), leftWidth = leftWidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE, right.attributes.RESOLUTION && right.attributes.RESOLUTION.width && (rightWidth = right.attributes.RESOLUTION.width), leftWidth === (rightWidth = rightWidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE) && left.attributes.BANDWIDTH && right.attributes.BANDWIDTH) ? left.attributes.BANDWIDTH - right.attributes.BANDWIDTH : leftWidth - rightWidth;
|
||||
return (left.attributes.RESOLUTION && left.attributes.RESOLUTION.width && (leftWidth = left.attributes.RESOLUTION.width), leftWidth = leftWidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE, right.attributes.RESOLUTION && right.attributes.RESOLUTION.width && (rightWidth = right.attributes.RESOLUTION.width), rightWidth = rightWidth || global_window__WEBPACK_IMPORTED_MODULE_0___default().Number.MAX_VALUE, leftWidth === rightWidth && left.attributes.BANDWIDTH && right.attributes.BANDWIDTH) ? left.attributes.BANDWIDTH - right.attributes.BANDWIDTH : leftWidth - rightWidth;
|
||||
},
|
||||
xhr: xhrFactory()
|
||||
};
|
||||
|
@ -71,8 +71,8 @@
|
||||
return Number(number);
|
||||
}), numberToBytes = function(number, _temp2) {
|
||||
var _ref2$le = (void 0 === _temp2 ? {} : _temp2).le, le = void 0 !== _ref2$le && _ref2$le;
|
||||
("bigint" != typeof number && "number" != typeof number || "number" == typeof number && number != number) && (number = 0);
|
||||
for(var byteCount = Math.ceil((number = BigInt(number)).toString(2).length / 8), bytes = new Uint8Array(new ArrayBuffer(byteCount)), i = 0; i < byteCount; i++){
|
||||
("bigint" != typeof number && "number" != typeof number || "number" == typeof number && number != number) && (number = 0), number = BigInt(number);
|
||||
for(var byteCount = Math.ceil(number.toString(2).length / 8), bytes = new Uint8Array(new ArrayBuffer(byteCount)), i = 0; i < byteCount; i++){
|
||||
var byteIndex = le ? i : Math.abs(i + 1 - bytes.length);
|
||||
bytes[byteIndex] = Number(number / BYTE_TABLE[i] & BigInt(0xff)), number < 0 && (bytes[byteIndex] = Math.abs(~bytes[byteIndex]), bytes[byteIndex] -= 0 === i ? 1 : 2);
|
||||
}
|
||||
@ -3583,7 +3583,7 @@
|
||||
}));
|
||||
var adaptationSetAttributes1, adaptationSetBaseUrls1, adaptationSetSegmentInfo, segmentInfo = getSegmentInformation(adaptationSet), representations = findChildren(adaptationSet, "Representation"), adaptationSetSegmentInfo1 = merge1(periodSegmentInfo, segmentInfo);
|
||||
return flatten(representations.map((adaptationSetAttributes1 = attrs, adaptationSetBaseUrls1 = adaptationSetBaseUrls, adaptationSetSegmentInfo = adaptationSetSegmentInfo1, function(representation) {
|
||||
var repBaseUrls = buildBaseUrls(adaptationSetBaseUrls1, findChildren(representation, "BaseURL")), attributes = merge1(adaptationSetAttributes1, parseAttributes(representation)), representationSegmentInfo = getSegmentInformation(representation);
|
||||
var repBaseUrlElements = findChildren(representation, "BaseURL"), repBaseUrls = buildBaseUrls(adaptationSetBaseUrls1, repBaseUrlElements), attributes = merge1(adaptationSetAttributes1, parseAttributes(representation)), representationSegmentInfo = getSegmentInformation(representation);
|
||||
return repBaseUrls.map(function(baseUrl) {
|
||||
return {
|
||||
segmentInfo: merge1(adaptationSetSegmentInfo, representationSegmentInfo),
|
||||
@ -3629,8 +3629,8 @@
|
||||
return attributes;
|
||||
}, parse = function(manifestString, options) {
|
||||
void 0 === options && (options = {});
|
||||
var parsedManifestInfo = inheritAttributes(stringToMpdXml(manifestString), options);
|
||||
return toM3u8((0, parsedManifestInfo.representationInfo).map(generateSegments), parsedManifestInfo.locations, options.sidxMapping);
|
||||
var parsedManifestInfo = inheritAttributes(stringToMpdXml(manifestString), options), playlists = (0, parsedManifestInfo.representationInfo).map(generateSegments);
|
||||
return toM3u8(playlists, parsedManifestInfo.locations, options.sidxMapping);
|
||||
}, parseUTCTiming = function(manifestString) {
|
||||
return parseUTCTimingScheme(stringToMpdXml(manifestString));
|
||||
};
|
||||
|
@ -1,4 +1,4 @@
|
||||
export function log2(v) {
|
||||
var r, shift;
|
||||
return v >>>= r = (v > 0xffff) << 4, v >>>= shift = (v > 0xff) << 3, r |= shift, shift = (v > 0xf) << 2, v >>>= shift, r |= shift, shift = (v > 0x3) << 1, v >>>= shift, r |= shift, r | v >> 1;
|
||||
return r = (v > 0xffff) << 4, v >>>= r, shift = (v > 0xff) << 3, v >>>= shift, r |= shift, shift = (v > 0xf) << 2, v >>>= shift, r |= shift, shift = (v > 0x3) << 1, v >>>= shift, r |= shift, r | v >> 1;
|
||||
}
|
||||
|
@ -1329,7 +1329,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 3,
|
||||
mutation_by_call_count: 92,
|
||||
usage_count: 103,
|
||||
reassigned_with_assignment: false,
|
||||
@ -11941,7 +11941,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 3,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 1,
|
||||
reassigned_with_assignment: true,
|
||||
@ -29871,7 +29871,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 3,
|
||||
usage_count: 3,
|
||||
reassigned_with_assignment: false,
|
||||
@ -65899,7 +65899,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 3,
|
||||
mutation_by_call_count: 4,
|
||||
usage_count: 6,
|
||||
reassigned_with_assignment: true,
|
||||
@ -71137,7 +71137,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 3,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 5,
|
||||
reassigned_with_assignment: true,
|
||||
@ -78707,7 +78707,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: false,
|
||||
@ -78720,7 +78720,7 @@ TestSnapshot {
|
||||
used_above_decl: false,
|
||||
is_fn_local: true,
|
||||
used_by_nested_fn: true,
|
||||
executed_multiple_time: false,
|
||||
executed_multiple_time: true,
|
||||
used_in_cond: true,
|
||||
var_kind: Some(
|
||||
"var",
|
||||
@ -78747,7 +78747,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 1,
|
||||
reassigned_with_assignment: false,
|
||||
@ -79835,7 +79835,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 28,
|
||||
usage_count: 30,
|
||||
reassigned_with_assignment: false,
|
||||
@ -82267,12 +82267,12 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: true,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 8,
|
||||
reassigned_with_assignment: false,
|
||||
reassigned_with_var_decl: false,
|
||||
mutated: false,
|
||||
mutated: true,
|
||||
has_property_access: true,
|
||||
has_property_mutation: false,
|
||||
accessed_props: {},
|
||||
@ -83475,7 +83475,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 3,
|
||||
mutation_by_call_count: 21,
|
||||
usage_count: 31,
|
||||
reassigned_with_assignment: false,
|
||||
@ -84891,12 +84891,12 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 4,
|
||||
reassigned_with_assignment: false,
|
||||
reassigned_with_var_decl: false,
|
||||
mutated: false,
|
||||
mutated: true,
|
||||
has_property_access: true,
|
||||
has_property_mutation: false,
|
||||
accessed_props: {},
|
||||
@ -85009,7 +85009,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 3,
|
||||
reassigned_with_assignment: false,
|
||||
@ -87411,12 +87411,12 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: false,
|
||||
reassigned_with_var_decl: false,
|
||||
mutated: false,
|
||||
mutated: true,
|
||||
has_property_access: true,
|
||||
has_property_mutation: false,
|
||||
accessed_props: {},
|
||||
@ -96239,7 +96239,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: true,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 2,
|
||||
usage_count: 3,
|
||||
reassigned_with_assignment: false,
|
||||
@ -144137,7 +144137,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 3,
|
||||
usage_count: 4,
|
||||
reassigned_with_assignment: false,
|
||||
|
@ -227,7 +227,7 @@
|
||||
for(var i$6 = 0; i$6 < len; ++i$6)if (isNeutral.test(types[i$6])) {
|
||||
var end$1 = void 0;
|
||||
for(end$1 = i$6 + 1; end$1 < len && isNeutral.test(types[end$1]); ++end$1);
|
||||
for(var before = (i$6 ? types[i$6 - 1] : outerType) == "L", replace$1 = before == ((end$1 < len ? types[end$1] : outerType) == "L") ? before ? "L" : "R" : outerType, j$1 = i$6; j$1 < end$1; ++j$1)types[j$1] = replace$1;
|
||||
for(var before = (i$6 ? types[i$6 - 1] : outerType) == "L", after = (end$1 < len ? types[end$1] : outerType) == "L", replace$1 = before == after ? before ? "L" : "R" : outerType, j$1 = i$6; j$1 < end$1; ++j$1)types[j$1] = replace$1;
|
||||
i$6 = end$1 - 1;
|
||||
}
|
||||
for(var m, order = [], i$7 = 0; i$7 < len;)if (countsAsLeft.test(types[i$7])) {
|
||||
@ -1210,7 +1210,7 @@
|
||||
}
|
||||
function prepareMeasureForLine(cm, line) {
|
||||
var cm2, line2, lineN, view, built, lineN1 = lineNo1(line), view1 = findViewForLine(cm, lineN1);
|
||||
view1 && !view1.text ? view1 = null : view1 && view1.changes && (updateLineForChanges(cm, view1, lineN1, getDimensions(cm)), cm.curOp.forceUpdate = !0), view1 || (view1 = (cm2 = cm, lineN = lineNo1(line2 = visualLine(line2 = line)), (view = cm2.display.externalMeasured = new LineView(cm2.doc, line2, lineN)).lineN = lineN, built = view.built = buildLineContent(cm2, view), view.text = built.pre, removeChildrenAndAdd(cm2.display.lineMeasure, built.pre), view));
|
||||
view1 && !view1.text ? view1 = null : view1 && view1.changes && (updateLineForChanges(cm, view1, lineN1, getDimensions(cm)), cm.curOp.forceUpdate = !0), view1 || (view1 = (cm2 = cm, line2 = visualLine(line2 = line), lineN = lineNo1(line2), (view = cm2.display.externalMeasured = new LineView(cm2.doc, line2, lineN)).lineN = lineN, built = view.built = buildLineContent(cm2, view), view.text = built.pre, removeChildrenAndAdd(cm2.display.lineMeasure, built.pre), view));
|
||||
var info = mapFromLineView(view1, line, lineN1);
|
||||
return {
|
||||
line: line,
|
||||
@ -1451,7 +1451,7 @@
|
||||
var coords = cursorCoords(cm, Pos(lineNo, ch2, sticky), "line", lineObj, preparedMeasure);
|
||||
baseX = coords.left, outside = y < coords.top ? -1 : y >= coords.bottom ? 1 : 0;
|
||||
}
|
||||
return PosWithInfo(lineNo, ch2 = skipExtendingChars(lineObj.text, ch2, 1), sticky, outside, x - baseX);
|
||||
return ch2 = skipExtendingChars(lineObj.text, ch2, 1), PosWithInfo(lineNo, ch2, sticky, outside, x - baseX);
|
||||
}
|
||||
function coordsBidiPart(cm, lineObj, lineNo, preparedMeasure, order, x, y) {
|
||||
var index = findFirst(function(i) {
|
||||
@ -3060,7 +3060,7 @@
|
||||
}, TextMarker.prototype.changed = function() {
|
||||
var this$1 = this, pos = this.find(-1, !0), widget = this, cm = this.doc.cm;
|
||||
pos && cm && runInOp(cm, function() {
|
||||
var line = pos.line, view = findViewForLine(cm, lineNo1(pos.line));
|
||||
var line = pos.line, lineN = lineNo1(pos.line), view = findViewForLine(cm, lineN);
|
||||
if (view && (clearLineMeasurementCacheFor(view), cm.curOp.selectionChanged = cm.curOp.forceUpdate = !0), cm.curOp.updateMaxLine = !0, !lineIsHidden(widget.doc, line) && null != widget.height) {
|
||||
var oldHeight = widget.height;
|
||||
widget.height = null;
|
||||
@ -3393,7 +3393,7 @@
|
||||
shared: options && options.shared,
|
||||
handleMouseEvents: options && options.handleMouseEvents
|
||||
};
|
||||
return markText(this, pos = clipPos(this, pos), pos, realOpts, "bookmark");
|
||||
return pos = clipPos(this, pos), markText(this, pos, pos, realOpts, "bookmark");
|
||||
},
|
||||
findMarksAt: function(pos) {
|
||||
pos = clipPos(this, pos);
|
||||
@ -5307,17 +5307,17 @@
|
||||
},
|
||||
getStateAfter: function(line, precise) {
|
||||
var doc = this.doc;
|
||||
return getContextBefore(this, (line = clipLine(doc, null == line ? doc.first + doc.size - 1 : line)) + 1, precise).state;
|
||||
return line = clipLine(doc, null == line ? doc.first + doc.size - 1 : line), getContextBefore(this, line + 1, precise).state;
|
||||
},
|
||||
cursorCoords: function(start, mode) {
|
||||
var range = this.doc.sel.primary();
|
||||
return cursorCoords(this, null == start ? range.head : "object" == typeof start ? clipPos(this.doc, start) : start ? range.from() : range.to(), mode || "page");
|
||||
var pos, range = this.doc.sel.primary();
|
||||
return pos = null == start ? range.head : "object" == typeof start ? clipPos(this.doc, start) : start ? range.from() : range.to(), cursorCoords(this, pos, mode || "page");
|
||||
},
|
||||
charCoords: function(pos, mode) {
|
||||
return charCoords(this, clipPos(this.doc, pos), mode || "page");
|
||||
},
|
||||
coordsChar: function(coords, mode) {
|
||||
return coordsChar(this, (coords = fromCoordSystem(this, coords, mode || "page")).left, coords.top);
|
||||
return coords = fromCoordSystem(this, coords, mode || "page"), coordsChar(this, coords.left, coords.top);
|
||||
},
|
||||
lineAtHeight: function(height, mode) {
|
||||
return height = fromCoordSystem(this, {
|
||||
@ -5349,18 +5349,18 @@
|
||||
};
|
||||
},
|
||||
addWidget: function(pos, node, scroll, vert, horiz) {
|
||||
var cm, scrollPos, display = this.display, top = (pos = cursorCoords(this, clipPos(this.doc, pos))).bottom, left = pos.left;
|
||||
var cm, rect, scrollPos, display = this.display, top = (pos = cursorCoords(this, clipPos(this.doc, pos))).bottom, left = pos.left;
|
||||
if (node.style.position = "absolute", node.setAttribute("cm-ignore-events", "true"), this.display.input.setUneditable(node), display.sizer.appendChild(node), "over" == vert) top = pos.top;
|
||||
else if ("above" == vert || "near" == vert) {
|
||||
var vspace = Math.max(display.wrapper.clientHeight, this.doc.height), hspace = Math.max(display.sizer.clientWidth, display.lineSpace.clientWidth);
|
||||
("above" == vert || pos.bottom + node.offsetHeight > vspace) && pos.top > node.offsetHeight ? top = pos.top - node.offsetHeight : pos.bottom + node.offsetHeight <= vspace && (top = pos.bottom), left + node.offsetWidth > hspace && (left = hspace - node.offsetWidth);
|
||||
}
|
||||
node.style.top = top + "px", node.style.left = node.style.right = "", "right" == horiz ? (left = display.sizer.clientWidth - node.offsetWidth, node.style.right = "0px") : ("left" == horiz ? left = 0 : "middle" == horiz && (left = (display.sizer.clientWidth - node.offsetWidth) / 2), node.style.left = left + "px"), scroll && (cm = this, null != (scrollPos = calculateScrollPos(cm, {
|
||||
node.style.top = top + "px", node.style.left = node.style.right = "", "right" == horiz ? (left = display.sizer.clientWidth - node.offsetWidth, node.style.right = "0px") : ("left" == horiz ? left = 0 : "middle" == horiz && (left = (display.sizer.clientWidth - node.offsetWidth) / 2), node.style.left = left + "px"), scroll && (cm = this, rect = {
|
||||
left: left,
|
||||
top: top,
|
||||
right: left + node.offsetWidth,
|
||||
bottom: top + node.offsetHeight
|
||||
})).scrollTop && updateScrollTop(cm, scrollPos.scrollTop), null != scrollPos.scrollLeft && setScrollLeft(cm, scrollPos.scrollLeft));
|
||||
}, null != (scrollPos = calculateScrollPos(cm, rect)).scrollTop && updateScrollTop(cm, scrollPos.scrollTop), null != scrollPos.scrollLeft && setScrollLeft(cm, scrollPos.scrollLeft));
|
||||
},
|
||||
triggerOnKeyDown: methodOp(onKeyDown),
|
||||
triggerOnKeyPress: methodOp(onKeyPress),
|
||||
|
@ -1770,7 +1770,7 @@
|
||||
},
|
||||
234: function(r28, t15, e22) {
|
||||
"use strict";
|
||||
var o4 = e22(219), n = e22(627), i = e22(749), a = i("Object.prototype.toString"), y = e22(449)(), p = y && "symbol" == typeof Symbol.toStringTag, f = n(), u = i("Array.prototype.indexOf", !0) || function(r, t) {
|
||||
var o4 = e22(219), n5 = e22(627), i = e22(749), a = i("Object.prototype.toString"), y = e22(449)(), p = y && "symbol" == typeof Symbol.toStringTag, f = n5(), u = i("Array.prototype.indexOf", !0) || function(r, t) {
|
||||
for(var e = 0; e < r.length; e += 1)if (r[e] === t) return e;
|
||||
return -1;
|
||||
}, s = i("String.prototype.slice"), c = {}, l = e22(982), d = Object.getPrototypeOf;
|
||||
@ -1778,7 +1778,11 @@
|
||||
var t = new __webpack_require__.g[r]();
|
||||
if (!(Symbol.toStringTag in t)) throw new EvalError("this engine has support for Symbol.toStringTag, but " + r + " does not have the property! Please report this.");
|
||||
var e = d(t), o = l(e, Symbol.toStringTag);
|
||||
o || (o = l(d(e), Symbol.toStringTag)), c[r] = o.get;
|
||||
if (!o) {
|
||||
var n = d(e);
|
||||
o = l(n, Symbol.toStringTag);
|
||||
}
|
||||
c[r] = o.get;
|
||||
});
|
||||
var g = function(r) {
|
||||
var t = !1;
|
||||
@ -1789,7 +1793,12 @@
|
||||
}), t;
|
||||
};
|
||||
r28.exports = function(r) {
|
||||
return !!r && "object" == typeof r && (p ? !!l && g(r) : u(f, s(a(r), 8, -1)) > -1);
|
||||
if (!r || "object" != typeof r) return !1;
|
||||
if (!p) {
|
||||
var t = s(a(r), 8, -1);
|
||||
return u(f, t) > -1;
|
||||
}
|
||||
return !!l && g(r);
|
||||
};
|
||||
},
|
||||
982: function(r, t, e) {
|
||||
@ -1936,13 +1945,13 @@
|
||||
var o5 = Object.getOwnPropertyDescriptors || function(r) {
|
||||
for(var t = Object.keys(r), e = {}, o = 0; o < t.length; o++)e[t[o]] = Object.getOwnPropertyDescriptor(r, t[o]);
|
||||
return e;
|
||||
}, n5 = /%[sdj%]/g;
|
||||
}, n6 = /%[sdj%]/g;
|
||||
t17.format = function(r34) {
|
||||
if (!isString(r34)) {
|
||||
for(var t = [], e = 0; e < arguments.length; e++)t.push(inspect(arguments[e]));
|
||||
return t.join(" ");
|
||||
}
|
||||
for(var e = 1, o = arguments, i = o.length, a = String(r34).replace(n5, function(r) {
|
||||
for(var e = 1, o = arguments, i = o.length, a = String(r34).replace(n6, function(r) {
|
||||
if ("%%" === r) return "%";
|
||||
if (e >= i) return r;
|
||||
switch(r){
|
||||
@ -2036,9 +2045,9 @@
|
||||
function formatError(r) {
|
||||
return "[" + Error.prototype.toString.call(r) + "]";
|
||||
}
|
||||
function formatArray(r, t, e, o, n6) {
|
||||
function formatArray(r, t, e, o, n7) {
|
||||
for(var i = [], a = 0, y = t.length; a < y; ++a)hasOwnProperty(t, String(a)) ? i.push(formatProperty(r, t, e, o, String(a), !0)) : i.push("");
|
||||
return n6.forEach(function(n) {
|
||||
return n7.forEach(function(n) {
|
||||
n.match(/^\d+$/) || i.push(formatProperty(r, t, e, o, n, !0));
|
||||
}), i;
|
||||
}
|
||||
@ -2201,8 +2210,8 @@
|
||||
}
|
||||
t17.log = function() {
|
||||
var r, t;
|
||||
console.log("%s - %s", (t = [
|
||||
pad((r = new Date()).getHours()),
|
||||
console.log("%s - %s", (r = new Date(), t = [
|
||||
pad(r.getHours()),
|
||||
pad(r.getMinutes()),
|
||||
pad(r.getSeconds()),
|
||||
].join(":"), [
|
||||
@ -2275,13 +2284,17 @@
|
||||
},
|
||||
715: function(r41, t21, e24) {
|
||||
"use strict";
|
||||
var o7 = e24(219), n7 = e24(627), i = e24(749), a = i("Object.prototype.toString"), y = e24(449)(), p = y && "symbol" == typeof Symbol.toStringTag, f = n7(), u = i("String.prototype.slice"), s = {}, c = e24(850), l = Object.getPrototypeOf;
|
||||
var o7 = e24(219), n8 = e24(627), i = e24(749), a = i("Object.prototype.toString"), y = e24(449)(), p = y && "symbol" == typeof Symbol.toStringTag, f = n8(), u = i("String.prototype.slice"), s = {}, c = e24(850), l = Object.getPrototypeOf;
|
||||
p && c && l && o7(f, function(r) {
|
||||
if ("function" == typeof __webpack_require__.g[r]) {
|
||||
var t = new __webpack_require__.g[r]();
|
||||
if (!(Symbol.toStringTag in t)) throw new EvalError("this engine has support for Symbol.toStringTag, but " + r + " does not have the property! Please report this.");
|
||||
var e = l(t), o = c(e, Symbol.toStringTag);
|
||||
o || (o = c(l(e), Symbol.toStringTag)), s[r] = o.get;
|
||||
if (!o) {
|
||||
var n = l(e);
|
||||
o = c(n, Symbol.toStringTag);
|
||||
}
|
||||
s[r] = o.get;
|
||||
}
|
||||
});
|
||||
var d = function(r) {
|
||||
@ -2299,7 +2312,7 @@
|
||||
},
|
||||
227: function(r42, t22, e25) {
|
||||
"use strict";
|
||||
var o8, n8 = SyntaxError, a = TypeError, getEvalledConstructor = function(r) {
|
||||
var o8, n9 = SyntaxError, a = TypeError, getEvalledConstructor = function(r) {
|
||||
try {
|
||||
return Function('"use strict"; return (' + r + ").constructor;")();
|
||||
} catch (r43) {}
|
||||
@ -2376,7 +2389,7 @@
|
||||
"%String%": String,
|
||||
"%StringIteratorPrototype%": f6 ? u4(""[Symbol.iterator]()) : o8,
|
||||
"%Symbol%": f6 ? Symbol : o8,
|
||||
"%SyntaxError%": n8,
|
||||
"%SyntaxError%": n9,
|
||||
"%ThrowTypeError%": p4,
|
||||
"%TypedArray%": d3,
|
||||
"%TypeError%": a,
|
||||
@ -2618,7 +2631,7 @@
|
||||
value: i
|
||||
};
|
||||
}
|
||||
throw new n8("intrinsic " + r + " does not exist!");
|
||||
throw new n9("intrinsic " + r + " does not exist!");
|
||||
};
|
||||
r42.exports = function(r, t) {
|
||||
if ("string" != typeof r || 0 === r.length) throw new a("intrinsic name must be a non-empty string");
|
||||
|
@ -48,10 +48,10 @@
|
||||
uri: "",
|
||||
exports: exports,
|
||||
packaged: !0
|
||||
};
|
||||
exports = module2(function(module, callback) {
|
||||
}, req = function(module, callback) {
|
||||
return _require(moduleName, module, callback);
|
||||
}, exports, mod) || mod.exports, define.modules[moduleName] = exports, delete define.payloads[moduleName];
|
||||
};
|
||||
exports = module2(req, exports, mod) || mod.exports, define.modules[moduleName] = exports, delete define.payloads[moduleName];
|
||||
}
|
||||
module2 = define.modules[moduleName] = exports || module2;
|
||||
}
|
||||
@ -2574,7 +2574,7 @@
|
||||
} else this.line += this.showInvisibles ? endOfLine : bidiUtil.DOT;
|
||||
var size, session = this.session, shift = 0;
|
||||
this.line = this.line.replace(/\t|[\u1100-\u2029, \u202F-\uFFE6]/g, function(ch, i) {
|
||||
return "\t" === ch || session.isFullWidth(ch.charCodeAt(0)) ? (shift += (size = "\t" === ch ? session.getScreenTabSize(i + shift) : 2) - 1, lang.stringRepeat(bidiUtil.DOT, size)) : ch;
|
||||
return "\t" === ch || session.isFullWidth(ch.charCodeAt(0)) ? (size = "\t" === ch ? session.getScreenTabSize(i + shift) : 2, shift += size - 1, lang.stringRepeat(bidiUtil.DOT, size)) : ch;
|
||||
}), this.isRtlDir && (this.fontMetrics.$main.textContent = this.line.charAt(this.line.length - 1) == bidiUtil.DOT ? this.line.substr(0, this.line.length - 1) : this.line, this.rtlLineOffset = this.contentWidth - this.fontMetrics.$main.getBoundingClientRect().width);
|
||||
}, this.updateBidiMap = function() {
|
||||
var textCharTypes = [];
|
||||
@ -5540,12 +5540,14 @@
|
||||
column: pos.column + 1
|
||||
}, match = chr && chr.match(/([\(\[\{])|([\)\]\}])/)), !match) return null;
|
||||
var startRange = new Range(pos.row, pos.column - 1, pos.row, pos.column), bracketPos = match[1] ? this.$findClosingBracket(match[1], pos) : this.$findOpeningBracket(match[2], pos);
|
||||
return bracketPos ? [
|
||||
startRange,
|
||||
new Range(bracketPos.row, bracketPos.column, bracketPos.row, bracketPos.column + 1)
|
||||
] : [
|
||||
if (!bracketPos) return [
|
||||
startRange
|
||||
];
|
||||
var endRange = new Range(bracketPos.row, bracketPos.column, bracketPos.row, bracketPos.column + 1);
|
||||
return [
|
||||
startRange,
|
||||
endRange
|
||||
];
|
||||
}, this.$brackets = {
|
||||
")": "(",
|
||||
"(": ")",
|
||||
@ -6195,7 +6197,7 @@
|
||||
var line, column, docRow = 0, docColumn = 0, row = 0, rowLength = 0, rowCache = this.$screenRowCache, i = this.$getRowCacheIndex(rowCache, screenRow), l = rowCache.length;
|
||||
if (l && i >= 0) var row = rowCache[i], docRow = this.$docRowCache[i], doCache = screenRow > rowCache[l - 1];
|
||||
else var doCache = !l;
|
||||
for(var maxRow = this.getLength() - 1, foldLine = this.getNextFoldLine(docRow), foldStart = foldLine ? foldLine.start.row : 1 / 0; row <= screenRow && !(row + (rowLength = this.getRowLength(docRow)) > screenRow) && !(docRow >= maxRow);)row += rowLength, ++docRow > foldStart && (docRow = foldLine.end.row + 1, foldStart = (foldLine = this.getNextFoldLine(docRow, foldLine)) ? foldLine.start.row : 1 / 0), doCache && (this.$docRowCache.push(docRow), this.$screenRowCache.push(row));
|
||||
for(var maxRow = this.getLength() - 1, foldLine = this.getNextFoldLine(docRow), foldStart = foldLine ? foldLine.start.row : 1 / 0; row <= screenRow && (rowLength = this.getRowLength(docRow), !(row + rowLength > screenRow) && !(docRow >= maxRow));)row += rowLength, ++docRow > foldStart && (docRow = foldLine.end.row + 1, foldStart = (foldLine = this.getNextFoldLine(docRow, foldLine)) ? foldLine.start.row : 1 / 0), doCache && (this.$docRowCache.push(docRow), this.$screenRowCache.push(row));
|
||||
if (foldLine && foldLine.start.row <= docRow) line = this.getFoldDisplayLine(foldLine), docRow = foldLine.start.row;
|
||||
else {
|
||||
if (row + rowLength <= screenRow || docRow > maxRow) return {
|
||||
|
@ -1061,7 +1061,7 @@
|
||||
}
|
||||
var hd = null;
|
||||
function Xc(a, b, c, d) {
|
||||
if (hd = null, null !== (a = Vc(a = wb(d)))) {
|
||||
if (hd = null, a = wb(d), null !== (a = Vc(a))) {
|
||||
if (null === (b = Ub(a))) a = null;
|
||||
else if (13 === (c = b.tag)) {
|
||||
if (null !== (a = Vb(b))) return a;
|
||||
@ -1238,21 +1238,21 @@
|
||||
movementY: function(a) {
|
||||
return "movementY" in a ? a.movementY : wd;
|
||||
}
|
||||
}), Ad = qd(zd), Cd = qd(A({}, zd, {
|
||||
}), Ad = qd(zd), Bd = A({}, zd, {
|
||||
dataTransfer: 0
|
||||
})), Ed = qd(A({}, td, {
|
||||
}), Cd = qd(Bd), Dd = A({}, td, {
|
||||
relatedTarget: 0
|
||||
})), Gd = qd(A({}, rd, {
|
||||
}), Ed = qd(Dd), Fd = A({}, rd, {
|
||||
animationName: 0,
|
||||
elapsedTime: 0,
|
||||
pseudoElement: 0
|
||||
})), Id = qd(A({}, rd, {
|
||||
}), Gd = qd(Fd), Hd = A({}, rd, {
|
||||
clipboardData: function(a) {
|
||||
return "clipboardData" in a ? a.clipboardData : window.clipboardData;
|
||||
}
|
||||
})), Kd = qd(A({}, rd, {
|
||||
}), Id = qd(Hd), Jd = A({}, rd, {
|
||||
data: 0
|
||||
})), Ld = {
|
||||
}), Kd = qd(Jd), Ld = {
|
||||
Esc: "Escape",
|
||||
Spacebar: " ",
|
||||
Left: "ArrowLeft",
|
||||
@ -1315,7 +1315,7 @@
|
||||
function yd() {
|
||||
return Od;
|
||||
}
|
||||
var Qd = qd(A({}, td, {
|
||||
var Pd = A({}, td, {
|
||||
key: function(a) {
|
||||
if (a.key) {
|
||||
var b = Ld[a.key] || a.key;
|
||||
@ -1341,7 +1341,7 @@
|
||||
which: function(a) {
|
||||
return "keypress" === a.type ? nd(a) : "keydown" === a.type || "keyup" === a.type ? a.keyCode : 0;
|
||||
}
|
||||
})), Sd = qd(A({}, zd, {
|
||||
}), Qd = qd(Pd), Rd = A({}, zd, {
|
||||
pointerId: 0,
|
||||
width: 0,
|
||||
height: 0,
|
||||
@ -1352,7 +1352,7 @@
|
||||
twist: 0,
|
||||
pointerType: 0,
|
||||
isPrimary: 0
|
||||
})), Ud = qd(A({}, td, {
|
||||
}), Sd = qd(Rd), Td = A({}, td, {
|
||||
touches: 0,
|
||||
targetTouches: 0,
|
||||
changedTouches: 0,
|
||||
@ -1361,11 +1361,11 @@
|
||||
ctrlKey: 0,
|
||||
shiftKey: 0,
|
||||
getModifierState: yd
|
||||
})), Wd = qd(A({}, rd, {
|
||||
}), Ud = qd(Td), Vd = A({}, rd, {
|
||||
propertyName: 0,
|
||||
elapsedTime: 0,
|
||||
pseudoElement: 0
|
||||
})), Yd = qd(A({}, zd, {
|
||||
}), Wd = qd(Vd), Xd = A({}, zd, {
|
||||
deltaX: function(a) {
|
||||
return "deltaX" in a ? a.deltaX : "wheelDeltaX" in a ? -a.wheelDeltaX : 0;
|
||||
},
|
||||
@ -1374,7 +1374,7 @@
|
||||
},
|
||||
deltaZ: 0,
|
||||
deltaMode: 0
|
||||
})), Zd = [
|
||||
}), Yd = qd(Xd), Zd = [
|
||||
9,
|
||||
13,
|
||||
27,
|
||||
@ -1431,7 +1431,8 @@
|
||||
re(a, 0);
|
||||
}
|
||||
function se(a) {
|
||||
if (Va(te(a))) return a;
|
||||
var b = te(a);
|
||||
if (Va(b)) return a;
|
||||
}
|
||||
function ue(a, b) {
|
||||
if ("change" === a) return b;
|
||||
@ -2956,7 +2957,7 @@
|
||||
hasEagerState: !1,
|
||||
eagerState: null,
|
||||
next: null
|
||||
}, Di(a) ? Ei(b, c) : (Fi(a, b, c), null !== (a = Lg(a, d, c = Jg())) && Gi(a, b, d));
|
||||
}, Di(a) ? Ei(b, c) : (Fi(a, b, c), c = Jg(), null !== (a = Lg(a, d, c)) && Gi(a, b, d));
|
||||
}
|
||||
function ni(a, b, c) {
|
||||
var d = Kg(a), e = {
|
||||
@ -2974,7 +2975,7 @@
|
||||
var g = b.lastRenderedState, h = f(g, c);
|
||||
if (e.hasEagerState = !0, e.eagerState = h, Ge(h, g)) return;
|
||||
} catch (k) {} finally{}
|
||||
null !== (a = Lg(a, d, c = Jg())) && Gi(a, b, d);
|
||||
c = Jg(), null !== (a = Lg(a, d, c)) && Gi(a, b, d);
|
||||
}
|
||||
}
|
||||
function Di(a) {
|
||||
@ -3099,7 +3100,7 @@
|
||||
var a = $h(), b = P.identifierPrefix;
|
||||
if (I) {
|
||||
var c = Zg, d = Yg;
|
||||
b = ":" + b + "R" + (c = (d & ~(1 << 32 - nc(d) - 1)).toString(32) + c), 0 < (c = Rh++) && (b += "H" + c.toString(32)), b += ":";
|
||||
c = (d & ~(1 << 32 - nc(d) - 1)).toString(32) + c, b = ":" + b + "R" + c, 0 < (c = Rh++) && (b += "H" + c.toString(32)), b += ":";
|
||||
} else b = ":" + b + "r" + (c = Sh++).toString(32) + ":";
|
||||
return a.memoizedState = b;
|
||||
},
|
||||
@ -3120,12 +3121,14 @@
|
||||
},
|
||||
useDebugValue: wi,
|
||||
useDeferredValue: function(a) {
|
||||
return zi(ai(), M.memoizedState, a);
|
||||
var b = ai();
|
||||
return zi(b, M.memoizedState, a);
|
||||
},
|
||||
useTransition: function() {
|
||||
var a = ci(bi)[0], b = ai().memoizedState;
|
||||
return [
|
||||
ci(bi)[0],
|
||||
ai().memoizedState
|
||||
a,
|
||||
b
|
||||
];
|
||||
},
|
||||
useMutableSource: ei,
|
||||
@ -3152,9 +3155,10 @@
|
||||
return null === M ? b.memoizedState = a : zi(b, M.memoizedState, a);
|
||||
},
|
||||
useTransition: function() {
|
||||
var a = di(bi)[0], b = ai().memoizedState;
|
||||
return [
|
||||
di(bi)[0],
|
||||
ai().memoizedState
|
||||
a,
|
||||
b
|
||||
];
|
||||
},
|
||||
useMutableSource: ei,
|
||||
@ -3635,13 +3639,13 @@
|
||||
var g = b.stateNode, h = b.memoizedProps;
|
||||
g.props = h;
|
||||
var k = g.context, l = c.contextType;
|
||||
l = "object" == typeof l && null !== l ? ug(l) : Xf(b, l = Yf(c) ? Wf : H.current);
|
||||
"object" == typeof l && null !== l ? l = ug(l) : (l = Yf(c) ? Wf : H.current, l = Xf(b, l));
|
||||
var n = c.getDerivedStateFromProps, u = "function" == typeof n || "function" == typeof g.getSnapshotBeforeUpdate;
|
||||
u || "function" != typeof g.UNSAFE_componentWillReceiveProps && "function" != typeof g.componentWillReceiveProps || (h !== d || k !== l) && Pg(b, g, d, l), wg = !1;
|
||||
var q = b.memoizedState;
|
||||
g.state = q, Eg(b, d, g, e), k = b.memoizedState, h !== d || q !== k || Vf.current || wg ? ("function" == typeof n && (Ig(b, c, n, d), k = b.memoizedState), (h = wg || Ng(b, c, h, d, q, k, l)) ? (u || "function" != typeof g.UNSAFE_componentWillMount && "function" != typeof g.componentWillMount || ("function" == typeof g.componentWillMount && g.componentWillMount(), "function" == typeof g.UNSAFE_componentWillMount && g.UNSAFE_componentWillMount()), "function" == typeof g.componentDidMount && (b.flags |= 4194308)) : ("function" == typeof g.componentDidMount && (b.flags |= 4194308), b.memoizedProps = d, b.memoizedState = k), g.props = d, g.state = k, g.context = l, d = h) : ("function" == typeof g.componentDidMount && (b.flags |= 4194308), d = !1);
|
||||
} else {
|
||||
g = b.stateNode, yg(a, b), h = b.memoizedProps, l = b.type === b.elementType ? h : kg(b.type, h), g.props = l, u = b.pendingProps, q = g.context, k = c.contextType, k = "object" == typeof k && null !== k ? ug(k) : Xf(b, k = Yf(c) ? Wf : H.current);
|
||||
g = b.stateNode, yg(a, b), h = b.memoizedProps, l = b.type === b.elementType ? h : kg(b.type, h), g.props = l, u = b.pendingProps, q = g.context, k = c.contextType, "object" == typeof k && null !== k ? k = ug(k) : (k = Yf(c) ? Wf : H.current, k = Xf(b, k));
|
||||
var y = c.getDerivedStateFromProps;
|
||||
(n = "function" == typeof y || "function" == typeof g.getSnapshotBeforeUpdate) || "function" != typeof g.UNSAFE_componentWillReceiveProps && "function" != typeof g.componentWillReceiveProps || (h !== u || q !== k) && Pg(b, g, d, k), wg = !1, q = b.memoizedState, g.state = q, Eg(b, d, g, e);
|
||||
var m = b.memoizedState;
|
||||
@ -4810,7 +4814,7 @@
|
||||
C = 1;
|
||||
var a17, b14, c7, h4 = W;
|
||||
W |= 4, lk.current = null, function(a, b) {
|
||||
if (Bf = cd, Me(a = Le())) {
|
||||
if (Bf = cd, a = Le(), Me(a)) {
|
||||
if ("selectionStart" in a) var c = {
|
||||
start: a.selectionStart,
|
||||
end: a.selectionEnd
|
||||
@ -5031,7 +5035,7 @@
|
||||
return !1;
|
||||
}
|
||||
function Wk(a, b, c) {
|
||||
b = Ki(a, b = Hi(c, b), 1), Ag(a, b), b = Jg(), a = Ak(a, 1), null !== a && (zc(a, 1, b), Ck(a, b));
|
||||
b = Hi(c, b), b = Ki(a, b, 1), Ag(a, b), b = Jg(), null !== (a = Ak(a, 1)) && (zc(a, 1, b), Ck(a, b));
|
||||
}
|
||||
function U(a, b, c) {
|
||||
if (3 === a.tag) Wk(a, a, c);
|
||||
@ -5043,7 +5047,7 @@
|
||||
if (1 === b.tag) {
|
||||
var d = b.stateNode;
|
||||
if ("function" == typeof b.type.getDerivedStateFromError || "function" == typeof d.componentDidCatch && (null === Oi || !Oi.has(d))) {
|
||||
a = Ni(b, a = Hi(c, a), 1), Ag(b, a), a = Jg(), b = Ak(b, 1), null !== b && (zc(b, 1, a), Ck(b, a));
|
||||
a = Hi(c, a), a = Ni(b, a, 1), Ag(b, a), a = Jg(), null !== (b = Ak(b, 1)) && (zc(b, 1, a), Ck(b, a));
|
||||
break;
|
||||
}
|
||||
}
|
||||
@ -5193,7 +5197,7 @@
|
||||
return b;
|
||||
}
|
||||
function dl(a, b, c, d, e, f, g, h, k) {
|
||||
return (a = al(c, d, !0, a, e, f, g, h, k)).context = cl(null), c = a.current, (f = zg(d = Jg(), e = Kg(c))).callback = null != b ? b : null, Ag(c, f), a.current.lanes = e, zc(a, e, d), Ck(a, d), a;
|
||||
return (a = al(c, d, !0, a, e, f, g, h, k)).context = cl(null), c = a.current, d = Jg(), e = Kg(c), (f = zg(d, e)).callback = null != b ? b : null, Ag(c, f), a.current.lanes = e, zc(a, e, d), Ck(a, d), a;
|
||||
}
|
||||
function el(a, b, c, d) {
|
||||
var e = b.current, f = Jg(), g = Kg(e);
|
||||
@ -5314,11 +5318,11 @@
|
||||
pendingSuspenseBoundaries: g.pendingSuspenseBoundaries,
|
||||
transitions: g.transitions
|
||||
}, b16.updateQueue.baseState = f, b16.memoizedState = f, 256 & b16.flags) {
|
||||
b16 = rj(a19, b16, d8, c9, e6 = Error(p(423)));
|
||||
e6 = Error(p(423)), b16 = rj(a19, b16, d8, c9, e6);
|
||||
break a;
|
||||
}
|
||||
if (d8 !== e6) {
|
||||
b16 = rj(a19, b16, d8, c9, e6 = Error(p(424)));
|
||||
e6 = Error(p(424)), b16 = rj(a19, b16, d8, c9, e6);
|
||||
break a;
|
||||
}
|
||||
for(eh = Kf(b16.stateNode.containerInfo.firstChild), dh = b16, I = !0, fh = null, c9 = zh(b16, null, d8, c9), b16.child = c9; c9;)c9.flags = -3 & c9.flags | 4096, c9 = c9.sibling;
|
||||
@ -5507,7 +5511,10 @@
|
||||
}), hl(a, 1);
|
||||
}
|
||||
}, Ec = function(a) {
|
||||
13 === a.tag && (Lg(a, 134217728, Jg()), hl(a, 134217728));
|
||||
if (13 === a.tag) {
|
||||
var b = Jg();
|
||||
Lg(a, 134217728, b), hl(a, 134217728);
|
||||
}
|
||||
}, Fc = function(a) {
|
||||
if (13 === a.tag) {
|
||||
var b = Jg(), c = Kg(a);
|
||||
|
File diff suppressed because one or more lines are too long
File diff suppressed because one or more lines are too long
@ -160,6 +160,9 @@ collapse_vars/issue_1537_destructuring_for_of/input.js
|
||||
collapse_vars/issue_1537_for_of/input.js
|
||||
collapse_vars/issue_1562/input.js
|
||||
collapse_vars/issue_1605_1/input.js
|
||||
collapse_vars/issue_1631_1/input.js
|
||||
collapse_vars/issue_1631_2/input.js
|
||||
collapse_vars/issue_1631_3/input.js
|
||||
collapse_vars/issue_2187_1/input.js
|
||||
collapse_vars/issue_2187_3/input.js
|
||||
collapse_vars/issue_2203_1/input.js
|
||||
|
@ -113,7 +113,7 @@
|
||||
function isScope(obj) {
|
||||
return obj && obj.$evalAsync && obj.$watch;
|
||||
}
|
||||
isNaN(msie = int((/msie (\d+)/.exec(lowercase(navigator.userAgent)) || [])[1])) && (msie = int((/trident\/.*; rv:(\d+)/.exec(lowercase(navigator.userAgent)) || [])[1])), noop.$inject = [], identity.$inject = [];
|
||||
msie = int((/msie (\d+)/.exec(lowercase(navigator.userAgent)) || [])[1]), isNaN(msie) && (msie = int((/trident\/.*; rv:(\d+)/.exec(lowercase(navigator.userAgent)) || [])[1])), noop.$inject = [], identity.$inject = [];
|
||||
var trim1 = String.prototype.trim ? function(value) {
|
||||
return isString(value) ? value.trim() : value;
|
||||
} : function(value) {
|
||||
@ -230,7 +230,7 @@
|
||||
function parseKeyValue(keyValue1) {
|
||||
var key_value, key, obj = {};
|
||||
return forEach((keyValue1 || "").split("&"), function(keyValue) {
|
||||
if (keyValue && isDefined(key = tryDecodeURIComponent((key_value = keyValue.split("="))[0]))) {
|
||||
if (keyValue && (key = tryDecodeURIComponent((key_value = keyValue.split("="))[0]), isDefined(key))) {
|
||||
var val = !isDefined(key_value[1]) || tryDecodeURIComponent(key_value[1]);
|
||||
obj[key] ? isArray(obj[key]) ? obj[key].push(val) : obj[key] = [
|
||||
obj[key],
|
||||
@ -255,7 +255,10 @@
|
||||
}
|
||||
function bootstrap1(element1, modules) {
|
||||
var doBootstrap = function() {
|
||||
if ((element1 = jqLite(element1)).injector()) throw ngMinErr1("btstrpd", "App Already Bootstrapped with this Element '{0}'", element1[0] === document1 ? "document" : startingTag(element1));
|
||||
if ((element1 = jqLite(element1)).injector()) {
|
||||
var tag = element1[0] === document1 ? "document" : startingTag(element1);
|
||||
throw ngMinErr1("btstrpd", "App Already Bootstrapped with this Element '{0}'", tag);
|
||||
}
|
||||
(modules = modules || []).unshift([
|
||||
"$provide",
|
||||
function($provide) {
|
||||
@ -778,7 +781,7 @@
|
||||
invoke: invoke,
|
||||
instantiate: function(Type, locals) {
|
||||
var instance, returnedValue, Constructor = function() {};
|
||||
return Constructor.prototype = (isArray(Type) ? Type[Type.length - 1] : Type).prototype, isObject(returnedValue = invoke(Type, instance = new Constructor(), locals)) || isFunction(returnedValue) ? returnedValue : instance;
|
||||
return Constructor.prototype = (isArray(Type) ? Type[Type.length - 1] : Type).prototype, returnedValue = invoke(Type, instance = new Constructor(), locals), isObject(returnedValue) || isFunction(returnedValue) ? returnedValue : instance;
|
||||
},
|
||||
get: getService,
|
||||
annotate: annotate,
|
||||
@ -1131,7 +1134,7 @@
|
||||
}
|
||||
function groupElementsLinkFnWrapper(linkFn, attrStart, attrEnd) {
|
||||
return function(scope, element, attrs, controllers, transcludeFn) {
|
||||
return linkFn(scope, element = groupScan(element[0], attrStart, attrEnd), attrs, controllers, transcludeFn);
|
||||
return element = groupScan(element[0], attrStart, attrEnd), linkFn(scope, element, attrs, controllers, transcludeFn);
|
||||
};
|
||||
}
|
||||
function applyDirectivesToNode(directives, compileNode, templateAttrs, transcludeFn1, jqCollection, originalReplaceDirective, preLinkFns, postLinkFns, previousCompileContext) {
|
||||
@ -1433,7 +1436,7 @@
|
||||
function($injector, $window) {
|
||||
return function(expression, locals) {
|
||||
var instance, match, constructor, identifier;
|
||||
if (isString(expression) && (constructor = (match = expression.match(CNTRL_REG))[1], identifier = match[3], assertArgFn(expression = controllers.hasOwnProperty(constructor) ? controllers[constructor] : getter1(locals.$scope, constructor, !0) || getter1($window, constructor, !0), constructor, !0)), instance = $injector.instantiate(expression, locals), identifier) {
|
||||
if (isString(expression) && (constructor = (match = expression.match(CNTRL_REG))[1], identifier = match[3], expression = controllers.hasOwnProperty(constructor) ? controllers[constructor] : getter1(locals.$scope, constructor, !0) || getter1($window, constructor, !0), assertArgFn(expression, constructor, !0)), instance = $injector.instantiate(expression, locals), identifier) {
|
||||
if (!(locals && "object" == typeof locals.$scope)) throw minErr("$controller")("noscp", "Cannot export controller '{0}' as '{1}'! No $scope object provided via `locals`.", constructor || expression.name, identifier);
|
||||
locals.$scope[identifier] = instance;
|
||||
}
|
||||
@ -1533,7 +1536,7 @@
|
||||
});
|
||||
}
|
||||
var defHeaderName, lowercaseDefHeaderName, reqHeaderName, defHeaders = defaults.headers, reqHeaders = extend({}, config.headers);
|
||||
execHeaders(defHeaders = extend({}, defHeaders.common, defHeaders[lowercase(config.method)])), execHeaders(reqHeaders);
|
||||
defHeaders = extend({}, defHeaders.common, defHeaders[lowercase(config.method)]), execHeaders(defHeaders), execHeaders(reqHeaders);
|
||||
defaultHeadersIteration: for(defHeaderName in defHeaders){
|
||||
for(reqHeaderName in lowercaseDefHeaderName = lowercase(defHeaderName), reqHeaders)if (lowercase(reqHeaderName) === lowercaseDefHeaderName) continue defaultHeadersIteration;
|
||||
reqHeaders[defHeaderName] = defHeaders[defHeaderName];
|
||||
@ -1576,7 +1579,7 @@
|
||||
}), url + (-1 == url.indexOf("?") ? "?" : "&") + parts.join("&");
|
||||
}(config.url, config.params);
|
||||
if ($http.pendingRequests.push(config), promise.then(removePendingReq, removePendingReq), (config.cache || defaults.cache) && !1 !== config.cache && "GET" == config.method && (cache = isObject(config.cache) ? config.cache : isObject(defaults.cache) ? defaults.cache : defaultCache), cache) {
|
||||
if (isDefined(cachedResp = cache.get(url1))) {
|
||||
if (cachedResp = cache.get(url1), isDefined(cachedResp)) {
|
||||
if (cachedResp.then) return cachedResp.then(removePendingReq, removePendingReq), cachedResp;
|
||||
isArray(cachedResp) ? resolvePromise(cachedResp[1], cachedResp[0], copy(cachedResp[2])) : resolvePromise(cachedResp, 200, {});
|
||||
} else cache.put(url1, promise);
|
||||
@ -1728,7 +1731,8 @@
|
||||
for(var part, i = 0, ii = length; i < ii; i++)"function" == typeof (part = parts[i]) && (part = part(context), part = trustedContext ? $sce.getTrusted(trustedContext, part) : $sce.valueOf(part), null === part || isUndefined(part) ? part = "" : "string" != typeof part && (part = toJson(part))), concat[i] = part;
|
||||
return concat.join("");
|
||||
} catch (err) {
|
||||
$exceptionHandler($interpolateMinErr("interr", "Can't interpolate: {0}\n{1}", text, err.toString()));
|
||||
var newErr = $interpolateMinErr("interr", "Can't interpolate: {0}\n{1}", text, err.toString());
|
||||
$exceptionHandler(newErr);
|
||||
}
|
||||
}).exp = text, fn.parts = parts, fn;
|
||||
}
|
||||
@ -2154,7 +2158,9 @@
|
||||
return "-" === ch || "+" === ch || this.isNumber(ch);
|
||||
},
|
||||
throwError: function(error, start, end) {
|
||||
throw end = end || this.index, $parseMinErr("lexerr", "Lexer Error: {0} at column{1} in expression [{2}].", error, isDefined(start) ? "s " + start + "-" + this.index + " [" + this.text.substring(start, end) + "]" : " " + end, this.text);
|
||||
end = end || this.index;
|
||||
var colStr = isDefined(start) ? "s " + start + "-" + this.index + " [" + this.text.substring(start, end) + "]" : " " + end;
|
||||
throw $parseMinErr("lexerr", "Lexer Error: {0} at column{1} in expression [{2}].", error, colStr, this.text);
|
||||
},
|
||||
readNumber: function() {
|
||||
for(var number = "", start = this.index; this.index < this.text.length;){
|
||||
@ -2418,8 +2424,8 @@
|
||||
})), v = v.$$v), v;
|
||||
}, {
|
||||
assign: function(self, value, locals) {
|
||||
var key = indexFn(self, locals), safe = ensureSafeObject(obj(self, locals), parser.text);
|
||||
return safe[key] = value;
|
||||
var key = indexFn(self, locals);
|
||||
return ensureSafeObject(obj(self, locals), parser.text)[key] = value;
|
||||
}
|
||||
});
|
||||
},
|
||||
@ -2432,7 +2438,9 @@
|
||||
return function(scope, locals) {
|
||||
for(var args = [], context = contextGetter ? contextGetter(scope, locals) : scope, i = 0; i < argsFn.length; i++)args.push(argsFn[i](scope, locals));
|
||||
var fnPtr = fn(scope, locals, context) || noop;
|
||||
return ensureSafeObject(context, parser.text), ensureSafeObject(fnPtr, parser.text), ensureSafeObject(fnPtr.apply ? fnPtr.apply(context, args) : fnPtr(args[0], args[1], args[2], args[3], args[4]), parser.text);
|
||||
ensureSafeObject(context, parser.text), ensureSafeObject(fnPtr, parser.text);
|
||||
var v = fnPtr.apply ? fnPtr.apply(context, args) : fnPtr(args[0], args[1], args[2], args[3], args[4]);
|
||||
return ensureSafeObject(v, parser.text);
|
||||
};
|
||||
},
|
||||
arrayDeclaration: function() {
|
||||
@ -4213,7 +4221,7 @@
|
||||
} else selected = modelValue === valueFn(scope, locals);
|
||||
selectedSet = selectedSet || selected;
|
||||
}
|
||||
label = isDefined(label = displayFn(scope, locals)) ? label : "", optionGroup.push({
|
||||
label = displayFn(scope, locals), label = isDefined(label) ? label : "", optionGroup.push({
|
||||
id: trackFn ? trackFn(scope, locals) : keyName ? keys[index] : index,
|
||||
label: label,
|
||||
selected: selected
|
||||
|
@ -1610,7 +1610,7 @@
|
||||
var temp, i, elem, preMap = [], postMap = [], preexisting = results.length, elems = seed || multipleContexts(selector || "*", context.nodeType ? [
|
||||
context
|
||||
] : context, []), matcherIn = preFilter && (seed || !selector) ? condense(elems, preMap, preFilter, context, xml) : elems, matcherOut = matcher ? postFinder || (seed ? preFilter : preexisting || postFilter) ? [] : results : matcherIn;
|
||||
if (matcher && matcher(matcherIn, matcherOut, context, xml), postFilter) for(postFilter(temp = condense(matcherOut, postMap), [], context, xml), i = temp.length; i--;)(elem = temp[i]) && (matcherOut[postMap[i]] = !(matcherIn[postMap[i]] = elem));
|
||||
if (matcher && matcher(matcherIn, matcherOut, context, xml), postFilter) for(temp = condense(matcherOut, postMap), postFilter(temp, [], context, xml), i = temp.length; i--;)(elem = temp[i]) && (matcherOut[postMap[i]] = !(matcherIn[postMap[i]] = elem));
|
||||
if (seed) {
|
||||
if (postFinder || preFilter) {
|
||||
if (postFinder) {
|
||||
|
@ -568,7 +568,11 @@
|
||||
!error$1 || error$1 instanceof Error || (setCurrentlyValidatingElement(element), error1("%s: type specification of %s `%s` is invalid; the type checker function must return `null` or an `Error` but returned a %s. You may have forgotten to pass an argument to the type checker creator (arrayOf, instanceOf, objectOf, oneOf, oneOfType, and shape all require an argument).", componentName || "React class", location, typeSpecName, typeof error$1), setCurrentlyValidatingElement(null)), error$1 instanceof Error && !(error$1.message in loggedTypeFailures) && (loggedTypeFailures[error$1.message] = !0, setCurrentlyValidatingElement(element), error1("Failed %s type: %s", location, error$1.message), setCurrentlyValidatingElement(null));
|
||||
}
|
||||
}(propTypes, element1.props, "prop", name, element1);
|
||||
} else void 0 === type.PropTypes || propTypesMisspellWarningShown || (propTypesMisspellWarningShown = !0, error1("Component %s declared `PropTypes` instead of `propTypes`. Did you misspell the property assignment?", getComponentName(type) || "Unknown"));
|
||||
} else if (void 0 !== type.PropTypes && !propTypesMisspellWarningShown) {
|
||||
propTypesMisspellWarningShown = !0;
|
||||
var _name = getComponentName(type);
|
||||
error1("Component %s declared `PropTypes` instead of `propTypes`. Did you misspell the property assignment?", _name || "Unknown");
|
||||
}
|
||||
"function" != typeof type.getDefaultProps || type.getDefaultProps.isReactClassApproved || error1("getDefaultProps is only used on classic React.createClass definitions. Use a static property named `defaultProps` instead.");
|
||||
}
|
||||
}
|
||||
|
@ -2502,7 +2502,7 @@
|
||||
}
|
||||
}
|
||||
function attemptToDispatchEvent(domEventName, eventSystemFlags, targetContainer, nativeEvent) {
|
||||
var targetInst = getClosestInstanceFromNode(getEventTarget(nativeEvent));
|
||||
var nativeEventTarget = getEventTarget(nativeEvent), targetInst = getClosestInstanceFromNode(nativeEventTarget);
|
||||
if (null !== targetInst) {
|
||||
var nearestMounted = getNearestMountedFiber(targetInst);
|
||||
if (null === nearestMounted) targetInst = null;
|
||||
@ -2600,21 +2600,21 @@
|
||||
movementY: function(event) {
|
||||
return "movementY" in event ? event.movementY : lastMovementY;
|
||||
}
|
||||
}), SyntheticMouseEvent = createSyntheticEvent(MouseEventInterface), SyntheticDragEvent = createSyntheticEvent(_assign({}, MouseEventInterface, {
|
||||
}), SyntheticMouseEvent = createSyntheticEvent(MouseEventInterface), DragEventInterface = _assign({}, MouseEventInterface, {
|
||||
dataTransfer: 0
|
||||
})), SyntheticFocusEvent = createSyntheticEvent(_assign({}, UIEventInterface, {
|
||||
}), SyntheticDragEvent = createSyntheticEvent(DragEventInterface), FocusEventInterface = _assign({}, UIEventInterface, {
|
||||
relatedTarget: 0
|
||||
})), SyntheticAnimationEvent = createSyntheticEvent(_assign({}, EventInterface, {
|
||||
}), SyntheticFocusEvent = createSyntheticEvent(FocusEventInterface), AnimationEventInterface = _assign({}, EventInterface, {
|
||||
animationName: 0,
|
||||
elapsedTime: 0,
|
||||
pseudoElement: 0
|
||||
})), SyntheticClipboardEvent = createSyntheticEvent(_assign({}, EventInterface, {
|
||||
}), SyntheticAnimationEvent = createSyntheticEvent(AnimationEventInterface), ClipboardEventInterface = _assign({}, EventInterface, {
|
||||
clipboardData: function(event) {
|
||||
return "clipboardData" in event ? event.clipboardData : window.clipboardData;
|
||||
}
|
||||
})), SyntheticCompositionEvent = createSyntheticEvent(_assign({}, EventInterface, {
|
||||
}), SyntheticClipboardEvent = createSyntheticEvent(ClipboardEventInterface), CompositionEventInterface = _assign({}, EventInterface, {
|
||||
data: 0
|
||||
})), SyntheticInputEvent = SyntheticCompositionEvent, normalizeKey = {
|
||||
}), SyntheticCompositionEvent = createSyntheticEvent(CompositionEventInterface), SyntheticInputEvent = SyntheticCompositionEvent, normalizeKey = {
|
||||
Esc: "Escape",
|
||||
Spacebar: " ",
|
||||
Left: "ArrowLeft",
|
||||
@ -2679,7 +2679,7 @@
|
||||
function getEventModifierState(nativeEvent) {
|
||||
return modifierStateGetter;
|
||||
}
|
||||
var SyntheticKeyboardEvent = createSyntheticEvent(_assign({}, UIEventInterface, {
|
||||
var KeyboardEventInterface = _assign({}, UIEventInterface, {
|
||||
key: function(nativeEvent) {
|
||||
if (nativeEvent.key) {
|
||||
var key = normalizeKey[nativeEvent.key] || nativeEvent.key;
|
||||
@ -2709,7 +2709,7 @@
|
||||
which: function(event) {
|
||||
return "keypress" === event.type ? getEventCharCode(event) : "keydown" === event.type || "keyup" === event.type ? event.keyCode : 0;
|
||||
}
|
||||
})), SyntheticPointerEvent = createSyntheticEvent(_assign({}, MouseEventInterface, {
|
||||
}), SyntheticKeyboardEvent = createSyntheticEvent(KeyboardEventInterface), PointerEventInterface = _assign({}, MouseEventInterface, {
|
||||
pointerId: 0,
|
||||
width: 0,
|
||||
height: 0,
|
||||
@ -2720,7 +2720,7 @@
|
||||
twist: 0,
|
||||
pointerType: 0,
|
||||
isPrimary: 0
|
||||
})), SyntheticTouchEvent = createSyntheticEvent(_assign({}, UIEventInterface, {
|
||||
}), SyntheticPointerEvent = createSyntheticEvent(PointerEventInterface), TouchEventInterface = _assign({}, UIEventInterface, {
|
||||
touches: 0,
|
||||
targetTouches: 0,
|
||||
changedTouches: 0,
|
||||
@ -2729,11 +2729,11 @@
|
||||
ctrlKey: 0,
|
||||
shiftKey: 0,
|
||||
getModifierState: getEventModifierState
|
||||
})), SyntheticTransitionEvent = createSyntheticEvent(_assign({}, EventInterface, {
|
||||
}), SyntheticTouchEvent = createSyntheticEvent(TouchEventInterface), TransitionEventInterface = _assign({}, EventInterface, {
|
||||
propertyName: 0,
|
||||
elapsedTime: 0,
|
||||
pseudoElement: 0
|
||||
})), SyntheticWheelEvent = createSyntheticEvent(_assign({}, MouseEventInterface, {
|
||||
}), SyntheticTransitionEvent = createSyntheticEvent(TransitionEventInterface), WheelEventInterface = _assign({}, MouseEventInterface, {
|
||||
deltaX: function(event) {
|
||||
return "deltaX" in event ? event.deltaX : "wheelDeltaX" in event ? -event.wheelDeltaX : 0;
|
||||
},
|
||||
@ -2742,7 +2742,7 @@
|
||||
},
|
||||
deltaZ: 0,
|
||||
deltaMode: 0
|
||||
})), END_KEYCODES = [
|
||||
}), SyntheticWheelEvent = createSyntheticEvent(WheelEventInterface), END_KEYCODES = [
|
||||
9,
|
||||
13,
|
||||
27,
|
||||
@ -2808,7 +2808,8 @@
|
||||
processDispatchQueue(dispatchQueue, 0);
|
||||
}
|
||||
function getInstIfValueChanged(targetInst) {
|
||||
if (updateValueIfChanged(getNodeFromInstance(targetInst))) return targetInst;
|
||||
var targetNode = getNodeFromInstance(targetInst);
|
||||
if (updateValueIfChanged(targetNode)) return targetInst;
|
||||
}
|
||||
function getTargetInstForChangeEvent(domEventName, targetInst) {
|
||||
if ("change" === domEventName) return targetInst;
|
||||
@ -4133,7 +4134,8 @@
|
||||
if (instance && instance.__reactInternalMemoizedUnmaskedChildContext === unmaskedContext) return instance.__reactInternalMemoizedMaskedChildContext;
|
||||
var context = {};
|
||||
for(var key in contextTypes)context[key] = unmaskedContext[key];
|
||||
return checkPropTypes(contextTypes, context, "context", getComponentName(type) || "Unknown"), instance && cacheContext(workInProgress, unmaskedContext, context), context;
|
||||
var name = getComponentName(type) || "Unknown";
|
||||
return checkPropTypes(contextTypes, context, "context", name), instance && cacheContext(workInProgress, unmaskedContext, context), context;
|
||||
}
|
||||
function hasContextChanged() {
|
||||
return didPerformWorkStackCursor.current;
|
||||
@ -4160,7 +4162,8 @@
|
||||
}
|
||||
var childContext = instance.getChildContext();
|
||||
for(var contextKey in childContext)if (!(contextKey in childContextTypes)) throw Error((getComponentName(type) || "Unknown") + '.getChildContext(): key "' + contextKey + '" is not defined in childContextTypes.');
|
||||
return checkPropTypes(childContextTypes, childContext, "child context", getComponentName(type) || "Unknown"), _assign({}, parentContext, childContext);
|
||||
var name = getComponentName(type) || "Unknown";
|
||||
return checkPropTypes(childContextTypes, childContext, "child context", name), _assign({}, parentContext, childContext);
|
||||
}
|
||||
function pushContextProvider(workInProgress) {
|
||||
var instance = workInProgress.stateNode, memoizedMergedChildContext = instance && instance.__reactInternalMemoizedMergedChildContext || emptyContextObject;
|
||||
@ -4212,10 +4215,12 @@
|
||||
}
|
||||
}
|
||||
function runWithPriority$1(reactPriorityLevel, fn) {
|
||||
return Scheduler_runWithPriority(reactPriorityToSchedulerPriority(reactPriorityLevel), fn);
|
||||
var priorityLevel = reactPriorityToSchedulerPriority(reactPriorityLevel);
|
||||
return Scheduler_runWithPriority(priorityLevel, fn);
|
||||
}
|
||||
function scheduleCallback(reactPriorityLevel, callback, options) {
|
||||
return Scheduler_scheduleCallback(reactPriorityToSchedulerPriority(reactPriorityLevel), callback, options);
|
||||
var priorityLevel = reactPriorityToSchedulerPriority(reactPriorityLevel);
|
||||
return Scheduler_scheduleCallback(priorityLevel, callback, options);
|
||||
}
|
||||
function cancelCallback(callbackNode) {
|
||||
callbackNode !== fakeCallbackNode && Scheduler_cancelCallback(callbackNode);
|
||||
@ -4265,7 +4270,7 @@
|
||||
ReactStrictModeWarnings.recordUnsafeLifecycleWarnings = function(fiber, instance) {
|
||||
!didWarnAboutUnsafeLifecycles.has(fiber.type) && ("function" == typeof instance.componentWillMount && !0 !== instance.componentWillMount.__suppressDeprecationWarning && pendingComponentWillMountWarnings.push(fiber), 1 & fiber.mode && "function" == typeof instance.UNSAFE_componentWillMount && pendingUNSAFE_ComponentWillMountWarnings.push(fiber), "function" == typeof instance.componentWillReceiveProps && !0 !== instance.componentWillReceiveProps.__suppressDeprecationWarning && pendingComponentWillReceivePropsWarnings.push(fiber), 1 & fiber.mode && "function" == typeof instance.UNSAFE_componentWillReceiveProps && pendingUNSAFE_ComponentWillReceivePropsWarnings.push(fiber), "function" == typeof instance.componentWillUpdate && !0 !== instance.componentWillUpdate.__suppressDeprecationWarning && pendingComponentWillUpdateWarnings.push(fiber), 1 & fiber.mode && "function" == typeof instance.UNSAFE_componentWillUpdate && pendingUNSAFE_ComponentWillUpdateWarnings.push(fiber));
|
||||
}, ReactStrictModeWarnings.flushPendingUnsafeLifecycleWarnings = function() {
|
||||
var componentWillMountUniqueNames = new Set();
|
||||
var sortedNames, _sortedNames, _sortedNames2, _sortedNames3, _sortedNames4, _sortedNames5, componentWillMountUniqueNames = new Set();
|
||||
pendingComponentWillMountWarnings.length > 0 && (pendingComponentWillMountWarnings.forEach(function(fiber) {
|
||||
componentWillMountUniqueNames.add(getComponentName(fiber.type) || "Component"), didWarnAboutUnsafeLifecycles.add(fiber.type);
|
||||
}), pendingComponentWillMountWarnings = []);
|
||||
@ -4286,9 +4291,26 @@
|
||||
componentWillUpdateUniqueNames.add(getComponentName(fiber.type) || "Component"), didWarnAboutUnsafeLifecycles.add(fiber.type);
|
||||
}), pendingComponentWillUpdateWarnings = []);
|
||||
var UNSAFE_componentWillUpdateUniqueNames = new Set();
|
||||
pendingUNSAFE_ComponentWillUpdateWarnings.length > 0 && (pendingUNSAFE_ComponentWillUpdateWarnings.forEach(function(fiber) {
|
||||
if (pendingUNSAFE_ComponentWillUpdateWarnings.length > 0 && (pendingUNSAFE_ComponentWillUpdateWarnings.forEach(function(fiber) {
|
||||
UNSAFE_componentWillUpdateUniqueNames.add(getComponentName(fiber.type) || "Component"), didWarnAboutUnsafeLifecycles.add(fiber.type);
|
||||
}), pendingUNSAFE_ComponentWillUpdateWarnings = []), UNSAFE_componentWillMountUniqueNames.size > 0 && error1("Using UNSAFE_componentWillMount in strict mode is not recommended and may indicate bugs in your code. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move code with side effects to componentDidMount, and set initial state in the constructor.\n\nPlease update the following components: %s", setToSortedString(UNSAFE_componentWillMountUniqueNames)), UNSAFE_componentWillReceivePropsUniqueNames.size > 0 && error1("Using UNSAFE_componentWillReceiveProps in strict mode is not recommended and may indicate bugs in your code. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n* If you're updating state whenever props change, refactor your code to use memoization techniques or move it to static getDerivedStateFromProps. Learn more at: https://reactjs.org/link/derived-state\n\nPlease update the following components: %s", setToSortedString(UNSAFE_componentWillReceivePropsUniqueNames)), UNSAFE_componentWillUpdateUniqueNames.size > 0 && error1("Using UNSAFE_componentWillUpdate in strict mode is not recommended and may indicate bugs in your code. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n\nPlease update the following components: %s", setToSortedString(UNSAFE_componentWillUpdateUniqueNames)), componentWillMountUniqueNames.size > 0 && warn("componentWillMount has been renamed, and is not recommended for use. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move code with side effects to componentDidMount, and set initial state in the constructor.\n* Rename componentWillMount to UNSAFE_componentWillMount to suppress this warning in non-strict mode. In React 18.x, only the UNSAFE_ name will work. To rename all deprecated lifecycles to their new names, you can run `npx react-codemod rename-unsafe-lifecycles` in your project source folder.\n\nPlease update the following components: %s", setToSortedString(componentWillMountUniqueNames)), componentWillReceivePropsUniqueNames.size > 0 && warn("componentWillReceiveProps has been renamed, and is not recommended for use. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n* If you're updating state whenever props change, refactor your code to use memoization techniques or move it to static getDerivedStateFromProps. Learn more at: https://reactjs.org/link/derived-state\n* Rename componentWillReceiveProps to UNSAFE_componentWillReceiveProps to suppress this warning in non-strict mode. In React 18.x, only the UNSAFE_ name will work. To rename all deprecated lifecycles to their new names, you can run `npx react-codemod rename-unsafe-lifecycles` in your project source folder.\n\nPlease update the following components: %s", setToSortedString(componentWillReceivePropsUniqueNames)), componentWillUpdateUniqueNames.size > 0 && warn("componentWillUpdate has been renamed, and is not recommended for use. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n* Rename componentWillUpdate to UNSAFE_componentWillUpdate to suppress this warning in non-strict mode. In React 18.x, only the UNSAFE_ name will work. To rename all deprecated lifecycles to their new names, you can run `npx react-codemod rename-unsafe-lifecycles` in your project source folder.\n\nPlease update the following components: %s", setToSortedString(componentWillUpdateUniqueNames));
|
||||
}), pendingUNSAFE_ComponentWillUpdateWarnings = []), UNSAFE_componentWillMountUniqueNames.size > 0) {
|
||||
error1("Using UNSAFE_componentWillMount in strict mode is not recommended and may indicate bugs in your code. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move code with side effects to componentDidMount, and set initial state in the constructor.\n\nPlease update the following components: %s", setToSortedString(UNSAFE_componentWillMountUniqueNames));
|
||||
}
|
||||
if (UNSAFE_componentWillReceivePropsUniqueNames.size > 0) {
|
||||
error1("Using UNSAFE_componentWillReceiveProps in strict mode is not recommended and may indicate bugs in your code. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n* If you're updating state whenever props change, refactor your code to use memoization techniques or move it to static getDerivedStateFromProps. Learn more at: https://reactjs.org/link/derived-state\n\nPlease update the following components: %s", setToSortedString(UNSAFE_componentWillReceivePropsUniqueNames));
|
||||
}
|
||||
if (UNSAFE_componentWillUpdateUniqueNames.size > 0) {
|
||||
error1("Using UNSAFE_componentWillUpdate in strict mode is not recommended and may indicate bugs in your code. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n\nPlease update the following components: %s", setToSortedString(UNSAFE_componentWillUpdateUniqueNames));
|
||||
}
|
||||
if (componentWillMountUniqueNames.size > 0) {
|
||||
warn("componentWillMount has been renamed, and is not recommended for use. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move code with side effects to componentDidMount, and set initial state in the constructor.\n* Rename componentWillMount to UNSAFE_componentWillMount to suppress this warning in non-strict mode. In React 18.x, only the UNSAFE_ name will work. To rename all deprecated lifecycles to their new names, you can run `npx react-codemod rename-unsafe-lifecycles` in your project source folder.\n\nPlease update the following components: %s", setToSortedString(componentWillMountUniqueNames));
|
||||
}
|
||||
if (componentWillReceivePropsUniqueNames.size > 0) {
|
||||
warn("componentWillReceiveProps has been renamed, and is not recommended for use. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n* If you're updating state whenever props change, refactor your code to use memoization techniques or move it to static getDerivedStateFromProps. Learn more at: https://reactjs.org/link/derived-state\n* Rename componentWillReceiveProps to UNSAFE_componentWillReceiveProps to suppress this warning in non-strict mode. In React 18.x, only the UNSAFE_ name will work. To rename all deprecated lifecycles to their new names, you can run `npx react-codemod rename-unsafe-lifecycles` in your project source folder.\n\nPlease update the following components: %s", setToSortedString(componentWillReceivePropsUniqueNames));
|
||||
}
|
||||
if (componentWillUpdateUniqueNames.size > 0) {
|
||||
warn("componentWillUpdate has been renamed, and is not recommended for use. See https://reactjs.org/link/unsafe-component-lifecycles for details.\n\n* Move data fetching code or side effects to componentDidUpdate.\n* Rename componentWillUpdate to UNSAFE_componentWillUpdate to suppress this warning in non-strict mode. In React 18.x, only the UNSAFE_ name will work. To rename all deprecated lifecycles to their new names, you can run `npx react-codemod rename-unsafe-lifecycles` in your project source folder.\n\nPlease update the following components: %s", setToSortedString(componentWillUpdateUniqueNames));
|
||||
}
|
||||
};
|
||||
var pendingLegacyContextWarning = new Map(), didWarnAboutLegacyContext = new Set();
|
||||
function resolveDefaultProps(Component, baseProps) {
|
||||
@ -5057,9 +5079,10 @@
|
||||
var container = 8 === nodeType ? rootContainerInstance.parentNode : rootContainerInstance;
|
||||
namespace = getChildNamespace(container.namespaceURI || null, type = container.tagName);
|
||||
}
|
||||
var ancestorInfo = updatedAncestorInfo(null, type.toLowerCase());
|
||||
return {
|
||||
namespace: namespace,
|
||||
ancestorInfo: updatedAncestorInfo(null, type.toLowerCase())
|
||||
ancestorInfo: ancestorInfo
|
||||
};
|
||||
}(nextRootInstance);
|
||||
pop(contextStackCursor$1, fiber), push(contextStackCursor$1, nextRootContext, fiber);
|
||||
@ -5432,9 +5455,16 @@
|
||||
source: source,
|
||||
subscribe: subscribe
|
||||
}, dispatcher.useEffect(function() {
|
||||
if (refs.getSnapshot = getSnapshot, refs.setSnapshot = setSnapshot, !objectIs(version, getVersion(source._source))) {
|
||||
refs.getSnapshot = getSnapshot, refs.setSnapshot = setSnapshot;
|
||||
var maybeNewVersion = getVersion(source._source);
|
||||
if (!objectIs(version, maybeNewVersion)) {
|
||||
var maybeNewSnapshot = getSnapshot(source._source);
|
||||
"function" == typeof maybeNewSnapshot && error1("Mutable source should not return a function as the snapshot value. Functions may close over mutable values and cause tearing."), objectIs(snapshot, maybeNewSnapshot) || (setSnapshot(maybeNewSnapshot), markRootMutableRead(root2, requestUpdateLane(fiber))), function(root, entangledLanes) {
|
||||
if ("function" == typeof maybeNewSnapshot && error1("Mutable source should not return a function as the snapshot value. Functions may close over mutable values and cause tearing."), !objectIs(snapshot, maybeNewSnapshot)) {
|
||||
setSnapshot(maybeNewSnapshot);
|
||||
var lane = requestUpdateLane(fiber);
|
||||
markRootMutableRead(root2, lane);
|
||||
}
|
||||
!function(root, entangledLanes) {
|
||||
root.entangledLanes |= entangledLanes;
|
||||
for(var entanglements = root.entanglements, lanes = entangledLanes; lanes > 0;){
|
||||
var index = pickArbitraryLaneIndex(lanes), lane = 1 << index;
|
||||
@ -5486,7 +5516,8 @@
|
||||
}, useMutableSource(hook, source, getSnapshot, subscribe);
|
||||
}
|
||||
function updateMutableSource(source, getSnapshot, subscribe) {
|
||||
return useMutableSource(updateWorkInProgressHook(), source, getSnapshot, subscribe);
|
||||
var hook = updateWorkInProgressHook();
|
||||
return useMutableSource(hook, source, getSnapshot, subscribe);
|
||||
}
|
||||
function mountState(initialState) {
|
||||
var hook = mountWorkInProgressHook();
|
||||
@ -5711,13 +5742,13 @@
|
||||
function mountOpaqueIdentifier() {
|
||||
var makeId = makeClientIdInDEV.bind(null, warnOnOpaqueIdentifierAccessInDEV.bind(null, currentlyRenderingFiber$1));
|
||||
if (isHydrating1) {
|
||||
var attemptToReadValue, didUpgrade = !1, fiber = currentlyRenderingFiber$1, id = {
|
||||
var attemptToReadValue, didUpgrade = !1, fiber = currentlyRenderingFiber$1, id = (attemptToReadValue = function() {
|
||||
throw didUpgrade || (didUpgrade = !0, isUpdatingOpaqueValueInRenderPhase = !0, setId(makeId()), isUpdatingOpaqueValueInRenderPhase = !1, warnOnOpaqueIdentifierAccessInDEV(fiber)), Error("The object passed back from useOpaqueIdentifier is meant to be passed through to attributes only. Do not read the value directly.");
|
||||
}, {
|
||||
$$typeof: REACT_OPAQUE_ID_TYPE,
|
||||
toString: attemptToReadValue = function() {
|
||||
throw didUpgrade || (didUpgrade = !0, isUpdatingOpaqueValueInRenderPhase = !0, setId(makeId()), isUpdatingOpaqueValueInRenderPhase = !1, warnOnOpaqueIdentifierAccessInDEV(fiber)), Error("The object passed back from useOpaqueIdentifier is meant to be passed through to attributes only. Do not read the value directly.");
|
||||
},
|
||||
toString: attemptToReadValue,
|
||||
valueOf: attemptToReadValue
|
||||
}, setId = mountState(id)[1];
|
||||
}), setId = mountState(id)[1];
|
||||
return (2 & currentlyRenderingFiber$1.mode) == 0 && (currentlyRenderingFiber$1.flags |= 512 | Update, pushEffect(5, function() {
|
||||
setId(makeId());
|
||||
}, void 0, null)), id;
|
||||
@ -6372,7 +6403,7 @@
|
||||
innerPropTypes && checkPropTypes(innerPropTypes, nextProps, "prop", getComponentName(Component));
|
||||
}
|
||||
var rendering2, unmaskedContext = getUnmaskedContext(workInProgress, Component, !0);
|
||||
if (context = getMaskedContext(workInProgress, unmaskedContext), prepareToReadContext(workInProgress, renderLanes), ReactCurrentOwner$1.current = workInProgress, rendering2 = !0, isRendering = rendering2, nextChildren = renderWithHooks(current, workInProgress, Component, nextProps, context, renderLanes), 1 & workInProgress.mode) {
|
||||
if (context = getMaskedContext(workInProgress, unmaskedContext), prepareToReadContext(workInProgress, renderLanes), ReactCurrentOwner$1.current = workInProgress, isRendering = !0, nextChildren = renderWithHooks(current, workInProgress, Component, nextProps, context, renderLanes), 1 & workInProgress.mode) {
|
||||
disableLogs();
|
||||
try {
|
||||
nextChildren = renderWithHooks(current, workInProgress, Component, nextProps, context, renderLanes);
|
||||
@ -6958,15 +6989,15 @@
|
||||
return fiberRoot.pendingContext && (fiberRoot.context = fiberRoot.pendingContext, fiberRoot.pendingContext = null), (null === current || null === current.child) && (popHydrationState(workInProgress) ? markUpdate(workInProgress) : fiberRoot.hydrate || (workInProgress.flags |= 256)), updateHostContainer(workInProgress), null;
|
||||
case 5:
|
||||
popHostContext(workInProgress);
|
||||
var rootContainerInstance = getRootHostContainer(), type12 = workInProgress.type;
|
||||
if (null !== current && null != workInProgress.stateNode) updateHostComponent$1(current, workInProgress, type12, newProps, rootContainerInstance), current.ref !== workInProgress.ref && markRef$1(workInProgress);
|
||||
var rootContainerInstance4 = getRootHostContainer(), type11 = workInProgress.type;
|
||||
if (null !== current && null != workInProgress.stateNode) updateHostComponent$1(current, workInProgress, type11, newProps, rootContainerInstance4), current.ref !== workInProgress.ref && markRef$1(workInProgress);
|
||||
else {
|
||||
if (!newProps) {
|
||||
if (!(null !== workInProgress.stateNode)) throw Error("We must have new props for new mounts. This error is likely caused by a bug in React. Please file an issue.");
|
||||
return null;
|
||||
}
|
||||
var currentHostContext = getHostContext();
|
||||
if (popHydrationState(workInProgress)) fiber = workInProgress, hostContext1 = currentHostContext, updatePayload1 = (instance = fiber.stateNode, type10 = fiber.type, props7 = fiber.memoizedProps, hostContext2 = hostContext1, internalInstanceHandle1 = fiber, precacheFiberNode(internalInstanceHandle1, instance), updateFiberProps(instance, props7), function(domElement, tag, rawProps, parentNamespace, rootContainerElement) {
|
||||
if (popHydrationState(workInProgress)) fiber = workInProgress, hostContext3 = currentHostContext, updatePayload1 = (instance = fiber.stateNode, type9 = fiber.type, props8 = fiber.memoizedProps, hostContext1 = hostContext3, internalInstanceHandle2 = fiber, precacheFiberNode(internalInstanceHandle2, instance), updateFiberProps(instance, props8), function(domElement, tag, rawProps, parentNamespace, rootContainerElement) {
|
||||
switch(suppressHydrationWarning = !0 === rawProps[SUPPRESS_HYDRATION_WARNING], isCustomComponentTag = isCustomComponent(tag, rawProps), validatePropertiesInDevelopment(tag, rawProps), tag){
|
||||
case "dialog":
|
||||
listenToNonDelegatedEvent("cancel", domElement), listenToNonDelegatedEvent("close", domElement);
|
||||
@ -7073,27 +7104,35 @@
|
||||
"function" == typeof rawProps.onClick && trapClickOnNonInteractiveElement(domElement);
|
||||
}
|
||||
return updatePayload;
|
||||
}(instance, type10, props7, hostContext2.namespace)), fiber.updateQueue = updatePayload1, null !== updatePayload1 && markUpdate(workInProgress);
|
||||
}(instance, type9, props8, hostContext1.namespace)), fiber.updateQueue = updatePayload1, null !== updatePayload1 && markUpdate(workInProgress);
|
||||
else {
|
||||
var type9, props9, rootContainerInstance1, hostContext, internalInstanceHandle, hostContextDev, domElement2, fiber, rootContainerInstance2, hostContext1, instance, type10, props7, hostContext2, internalInstanceHandle1, updatePayload1, domElement1, type11, props8, rootContainerInstance3, instance7 = (type9 = type12, props9 = newProps, rootContainerInstance1 = rootContainerInstance, hostContext = currentHostContext, internalInstanceHandle = workInProgress, hostContextDev = hostContext, validateDOMNesting(type9, null, hostContextDev.ancestorInfo), ("string" == typeof props9.children || "number" == typeof props9.children) && validateDOMNesting(null, "" + props9.children, updatedAncestorInfo(hostContextDev.ancestorInfo, type9)), domElement2 = function(type, props, rootContainerElement, parentNamespace) {
|
||||
var isCustomComponentTag, domElement, ownerDocument = getOwnerDocumentFromRootContainer(rootContainerElement), namespaceURI = parentNamespace;
|
||||
if (namespaceURI === HTML_NAMESPACE$1 && (namespaceURI = getIntrinsicNamespace(type)), namespaceURI === HTML_NAMESPACE$1) {
|
||||
if ((isCustomComponentTag = isCustomComponent(type, props)) || type === type.toLowerCase() || error1("<%s /> is using incorrect casing. Use PascalCase for React components, or lowercase for HTML elements.", type), "script" === type) {
|
||||
var div = ownerDocument.createElement("div");
|
||||
div.innerHTML = "<script></script>";
|
||||
var firstChild = div.firstChild;
|
||||
domElement = div.removeChild(firstChild);
|
||||
} else if ("string" == typeof props.is) domElement = ownerDocument.createElement(type, {
|
||||
is: props.is
|
||||
});
|
||||
else if (domElement = ownerDocument.createElement(type), "select" === type) {
|
||||
var node = domElement;
|
||||
props.multiple ? node.multiple = !0 : props.size && (node.size = props.size);
|
||||
}
|
||||
} else domElement = ownerDocument.createElementNS(namespaceURI, type);
|
||||
return namespaceURI !== HTML_NAMESPACE$1 || isCustomComponentTag || "[object HTMLUnknownElement]" !== Object.prototype.toString.call(domElement) || Object.prototype.hasOwnProperty.call(warnedUnknownTags, type) || (warnedUnknownTags[type] = !0, error1("The tag <%s> is unrecognized in this browser. If you meant to render a React component, start its name with an uppercase letter.", type)), domElement;
|
||||
}(type9, props9, rootContainerInstance1, hostContextDev.namespace), precacheFiberNode(internalInstanceHandle, domElement2), updateFiberProps(domElement2, props9), domElement2);
|
||||
appendAllChildren(instance7, workInProgress, !1, !1), workInProgress.stateNode = instance7, domElement1 = instance7, type11 = type12, function(domElement4, tag1, rawProps, rootContainerElement) {
|
||||
var fiber, rootContainerInstance1, hostContext3, instance, type9, props8, hostContext1, internalInstanceHandle2, updatePayload1, domElement1, type10, props7, rootContainerInstance2, instance7 = function(type12, props11, rootContainerInstance, hostContext, internalInstanceHandle) {
|
||||
var hostContextDev = hostContext;
|
||||
if (validateDOMNesting(type12, null, hostContextDev.ancestorInfo), "string" == typeof props11.children || "number" == typeof props11.children) {
|
||||
var string = "" + props11.children, ownAncestorInfo = updatedAncestorInfo(hostContextDev.ancestorInfo, type12);
|
||||
validateDOMNesting(null, string, ownAncestorInfo);
|
||||
}
|
||||
var domElement3 = function(type, props, rootContainerElement, parentNamespace) {
|
||||
var isCustomComponentTag, domElement, ownerDocument = getOwnerDocumentFromRootContainer(rootContainerElement), namespaceURI = parentNamespace;
|
||||
if (namespaceURI === HTML_NAMESPACE$1 && (namespaceURI = getIntrinsicNamespace(type)), namespaceURI === HTML_NAMESPACE$1) {
|
||||
if ((isCustomComponentTag = isCustomComponent(type, props)) || type === type.toLowerCase() || error1("<%s /> is using incorrect casing. Use PascalCase for React components, or lowercase for HTML elements.", type), "script" === type) {
|
||||
var div = ownerDocument.createElement("div");
|
||||
div.innerHTML = "<script></script>";
|
||||
var firstChild = div.firstChild;
|
||||
domElement = div.removeChild(firstChild);
|
||||
} else if ("string" == typeof props.is) domElement = ownerDocument.createElement(type, {
|
||||
is: props.is
|
||||
});
|
||||
else if (domElement = ownerDocument.createElement(type), "select" === type) {
|
||||
var node = domElement;
|
||||
props.multiple ? node.multiple = !0 : props.size && (node.size = props.size);
|
||||
}
|
||||
} else domElement = ownerDocument.createElementNS(namespaceURI, type);
|
||||
return namespaceURI !== HTML_NAMESPACE$1 || isCustomComponentTag || "[object HTMLUnknownElement]" !== Object.prototype.toString.call(domElement) || Object.prototype.hasOwnProperty.call(warnedUnknownTags, type) || (warnedUnknownTags[type] = !0, error1("The tag <%s> is unrecognized in this browser. If you meant to render a React component, start its name with an uppercase letter.", type)), domElement;
|
||||
}(type12, props11, rootContainerInstance, hostContextDev.namespace);
|
||||
return precacheFiberNode(internalInstanceHandle, domElement3), updateFiberProps(domElement3, props11), domElement3;
|
||||
}(type11, newProps, rootContainerInstance4, currentHostContext, workInProgress);
|
||||
appendAllChildren(instance7, workInProgress, !1, !1), workInProgress.stateNode = instance7, domElement1 = instance7, type10 = type11, function(domElement4, tag1, rawProps, rootContainerElement) {
|
||||
var element1, props13, node, value, props12, isCustomComponentTag1 = isCustomComponent(tag1, rawProps);
|
||||
switch(validatePropertiesInDevelopment(tag1, rawProps), tag1){
|
||||
case "dialog":
|
||||
@ -7165,7 +7204,7 @@
|
||||
default:
|
||||
"function" == typeof props12.onClick && trapClickOnNonInteractiveElement(domElement4);
|
||||
}
|
||||
}(domElement1, type11, props8 = newProps, rootContainerInstance), shouldAutoFocusHostComponent(type11, props8) && markUpdate(workInProgress);
|
||||
}(domElement1, type10, props7 = newProps, rootContainerInstance4), shouldAutoFocusHostComponent(type10, props7) && markUpdate(workInProgress);
|
||||
}
|
||||
null !== workInProgress.ref && markRef$1(workInProgress);
|
||||
}
|
||||
@ -7177,7 +7216,7 @@
|
||||
updateHostText$1(current, workInProgress, oldText, newText);
|
||||
} else {
|
||||
if ("string" != typeof newText && !(null !== workInProgress.stateNode)) throw Error("We must have new props for new mounts. This error is likely caused by a bug in React. Please file an issue.");
|
||||
var text8, rootContainerInstance4, hostContext3, internalInstanceHandle2, text4, rootContainerElement1, textNode1, _rootContainerInstance = getRootHostContainer(), _currentHostContext = getHostContext();
|
||||
var text8, rootContainerInstance3, hostContext2, internalInstanceHandle1, text4, rootContainerElement1, textNode1, _rootContainerInstance = getRootHostContainer(), _currentHostContext = getHostContext();
|
||||
popHydrationState(workInProgress) ? function(fiber) {
|
||||
var textInstance, text, internalInstanceHandle, textNode, text5, textInstance1 = fiber.stateNode, textContent = fiber.memoizedProps, shouldUpdate = (textInstance = textInstance1, text = textContent, precacheFiberNode(fiber, textInstance), textNode = textInstance, text5 = text, textNode.nodeValue !== text5);
|
||||
if (shouldUpdate) {
|
||||
@ -7193,7 +7232,7 @@
|
||||
}
|
||||
}
|
||||
return shouldUpdate;
|
||||
}(workInProgress) && markUpdate(workInProgress) : workInProgress.stateNode = (text8 = newText, rootContainerInstance4 = _rootContainerInstance, hostContext3 = _currentHostContext, internalInstanceHandle2 = workInProgress, validateDOMNesting(null, text8, hostContext3.ancestorInfo), precacheFiberNode(internalInstanceHandle2, textNode1 = (text4 = text8, getOwnerDocumentFromRootContainer(rootContainerInstance4).createTextNode(text4))), textNode1);
|
||||
}(workInProgress) && markUpdate(workInProgress) : workInProgress.stateNode = (text8 = newText, rootContainerInstance3 = _rootContainerInstance, hostContext2 = _currentHostContext, internalInstanceHandle1 = workInProgress, validateDOMNesting(null, text8, hostContext2.ancestorInfo), textNode1 = (text4 = text8, getOwnerDocumentFromRootContainer(rootContainerInstance3).createTextNode(text4)), precacheFiberNode(internalInstanceHandle1, textNode1), textNode1);
|
||||
}
|
||||
return null;
|
||||
case 13:
|
||||
@ -7364,64 +7403,70 @@
|
||||
}
|
||||
node.sibling.return = node.return, node = node.sibling;
|
||||
}
|
||||
}, updateHostContainer = function(workInProgress) {}, updateHostComponent$1 = function(current, workInProgress, type, newProps, rootContainerInstance) {
|
||||
var oldProps = current.memoizedProps;
|
||||
if (oldProps !== newProps) {
|
||||
var domElement5, type13, oldProps1, newProps3, rootContainerInstance5, hostContext, updatePayload3 = (domElement5 = workInProgress.stateNode, type13 = type, oldProps1 = oldProps, newProps3 = newProps, rootContainerInstance5 = rootContainerInstance, hostContext = getHostContext(), typeof newProps3.children != typeof oldProps1.children && ("string" == typeof newProps3.children || "number" == typeof newProps3.children) && validateDOMNesting(null, "" + newProps3.children, updatedAncestorInfo(hostContext.ancestorInfo, type13)), function(domElement, tag, lastRawProps, nextRawProps, rootContainerElement) {
|
||||
validatePropertiesInDevelopment(tag, nextRawProps);
|
||||
var lastProps, nextProps, propKey, styleName, updatePayload = null;
|
||||
switch(tag){
|
||||
case "input":
|
||||
lastProps = getHostProps(domElement, lastRawProps), nextProps = getHostProps(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
case "option":
|
||||
lastProps = getHostProps$1(domElement, lastRawProps), nextProps = getHostProps$1(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
case "select":
|
||||
lastProps = getHostProps$2(domElement, lastRawProps), nextProps = getHostProps$2(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
case "textarea":
|
||||
lastProps = getHostProps$3(domElement, lastRawProps), nextProps = getHostProps$3(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
default:
|
||||
lastProps = lastRawProps, nextProps = nextRawProps, "function" != typeof lastProps.onClick && "function" == typeof nextProps.onClick && trapClickOnNonInteractiveElement(domElement);
|
||||
}, updateHostContainer = function(workInProgress) {}, updateHostComponent$1 = function(current, workInProgress, type13, newProps3, rootContainerInstance) {
|
||||
var oldProps1 = current.memoizedProps;
|
||||
if (oldProps1 !== newProps3) {
|
||||
var instance = workInProgress.stateNode, currentHostContext = getHostContext(), updatePayload3 = function(domElement5, type, oldProps, newProps, rootContainerInstance, hostContext) {
|
||||
if (typeof newProps.children != typeof oldProps.children && ("string" == typeof newProps.children || "number" == typeof newProps.children)) {
|
||||
var string = "" + newProps.children, ownAncestorInfo = updatedAncestorInfo(hostContext.ancestorInfo, type);
|
||||
validateDOMNesting(null, string, ownAncestorInfo);
|
||||
}
|
||||
assertValidProps(tag, nextProps);
|
||||
var styleUpdates1 = null;
|
||||
for(propKey in lastProps)if (!nextProps.hasOwnProperty(propKey) && lastProps.hasOwnProperty(propKey) && null != lastProps[propKey]) {
|
||||
if (propKey === STYLE) {
|
||||
var lastStyle = lastProps[propKey];
|
||||
for(styleName in lastStyle)lastStyle.hasOwnProperty(styleName) && (styleUpdates1 || (styleUpdates1 = {}), styleUpdates1[styleName] = "");
|
||||
} else propKey !== DANGEROUSLY_SET_INNER_HTML && propKey !== CHILDREN && propKey !== SUPPRESS_CONTENT_EDITABLE_WARNING && propKey !== SUPPRESS_HYDRATION_WARNING && propKey !== AUTOFOCUS && (registrationNameDependencies1.hasOwnProperty(propKey) ? updatePayload || (updatePayload = []) : (updatePayload = updatePayload || []).push(propKey, null));
|
||||
}
|
||||
for(propKey in nextProps){
|
||||
var nextProp = nextProps[propKey], lastProp = null != lastProps ? lastProps[propKey] : void 0;
|
||||
if (nextProps.hasOwnProperty(propKey) && nextProp !== lastProp && (null != nextProp || null != lastProp)) {
|
||||
if (propKey === STYLE) {
|
||||
if (nextProp && Object.freeze(nextProp), lastProp) {
|
||||
for(styleName in lastProp)!lastProp.hasOwnProperty(styleName) || nextProp && nextProp.hasOwnProperty(styleName) || (styleUpdates1 || (styleUpdates1 = {}), styleUpdates1[styleName] = "");
|
||||
for(styleName in nextProp)nextProp.hasOwnProperty(styleName) && lastProp[styleName] !== nextProp[styleName] && (styleUpdates1 || (styleUpdates1 = {}), styleUpdates1[styleName] = nextProp[styleName]);
|
||||
} else styleUpdates1 || (updatePayload || (updatePayload = []), updatePayload.push(propKey, styleUpdates1)), styleUpdates1 = nextProp;
|
||||
} else if (propKey === DANGEROUSLY_SET_INNER_HTML) {
|
||||
var nextHtml = nextProp ? nextProp[HTML$1] : void 0, lastHtml = lastProp ? lastProp[HTML$1] : void 0;
|
||||
null != nextHtml && lastHtml !== nextHtml && (updatePayload = updatePayload || []).push(propKey, nextHtml);
|
||||
} else propKey === CHILDREN ? ("string" == typeof nextProp || "number" == typeof nextProp) && (updatePayload = updatePayload || []).push(propKey, "" + nextProp) : propKey !== SUPPRESS_CONTENT_EDITABLE_WARNING && propKey !== SUPPRESS_HYDRATION_WARNING && (registrationNameDependencies1.hasOwnProperty(propKey) ? (null != nextProp && ("function" != typeof nextProp && warnForInvalidEventListener(propKey, nextProp), "onScroll" === propKey && listenToNonDelegatedEvent("scroll", domElement)), updatePayload || lastProp === nextProp || (updatePayload = [])) : "object" == typeof nextProp && null !== nextProp && nextProp.$$typeof === REACT_OPAQUE_ID_TYPE ? nextProp.toString() : (updatePayload = updatePayload || []).push(propKey, nextProp));
|
||||
return function(domElement, tag, lastRawProps, nextRawProps, rootContainerElement) {
|
||||
validatePropertiesInDevelopment(tag, nextRawProps);
|
||||
var lastProps, nextProps, propKey, styleName, updatePayload = null;
|
||||
switch(tag){
|
||||
case "input":
|
||||
lastProps = getHostProps(domElement, lastRawProps), nextProps = getHostProps(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
case "option":
|
||||
lastProps = getHostProps$1(domElement, lastRawProps), nextProps = getHostProps$1(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
case "select":
|
||||
lastProps = getHostProps$2(domElement, lastRawProps), nextProps = getHostProps$2(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
case "textarea":
|
||||
lastProps = getHostProps$3(domElement, lastRawProps), nextProps = getHostProps$3(domElement, nextRawProps), updatePayload = [];
|
||||
break;
|
||||
default:
|
||||
lastProps = lastRawProps, nextProps = nextRawProps, "function" != typeof lastProps.onClick && "function" == typeof nextProps.onClick && trapClickOnNonInteractiveElement(domElement);
|
||||
}
|
||||
}
|
||||
return styleUpdates1 && (function(styleUpdates, nextStyles) {
|
||||
if (nextStyles) {
|
||||
var expandedUpdates = expandShorthandMap(styleUpdates), expandedStyles = expandShorthandMap(nextStyles), warnedAbout = {};
|
||||
for(var key in expandedUpdates){
|
||||
var originalKey = expandedUpdates[key], correctOriginalKey = expandedStyles[key];
|
||||
if (correctOriginalKey && originalKey !== correctOriginalKey) {
|
||||
var warningKey = originalKey + "," + correctOriginalKey;
|
||||
if (warnedAbout[warningKey]) continue;
|
||||
warnedAbout[warningKey] = !0, error1("%s a style property during rerender (%s) when a conflicting property is set (%s) can lead to styling bugs. To avoid this, don't mix shorthand and non-shorthand properties for the same value; instead, replace the shorthand with separate values.", isValueEmpty(styleUpdates[originalKey]) ? "Removing" : "Updating", originalKey, correctOriginalKey);
|
||||
}
|
||||
assertValidProps(tag, nextProps);
|
||||
var styleUpdates1 = null;
|
||||
for(propKey in lastProps)if (!nextProps.hasOwnProperty(propKey) && lastProps.hasOwnProperty(propKey) && null != lastProps[propKey]) {
|
||||
if (propKey === STYLE) {
|
||||
var lastStyle = lastProps[propKey];
|
||||
for(styleName in lastStyle)lastStyle.hasOwnProperty(styleName) && (styleUpdates1 || (styleUpdates1 = {}), styleUpdates1[styleName] = "");
|
||||
} else propKey !== DANGEROUSLY_SET_INNER_HTML && propKey !== CHILDREN && propKey !== SUPPRESS_CONTENT_EDITABLE_WARNING && propKey !== SUPPRESS_HYDRATION_WARNING && propKey !== AUTOFOCUS && (registrationNameDependencies1.hasOwnProperty(propKey) ? updatePayload || (updatePayload = []) : (updatePayload = updatePayload || []).push(propKey, null));
|
||||
}
|
||||
for(propKey in nextProps){
|
||||
var nextProp = nextProps[propKey], lastProp = null != lastProps ? lastProps[propKey] : void 0;
|
||||
if (nextProps.hasOwnProperty(propKey) && nextProp !== lastProp && (null != nextProp || null != lastProp)) {
|
||||
if (propKey === STYLE) {
|
||||
if (nextProp && Object.freeze(nextProp), lastProp) {
|
||||
for(styleName in lastProp)!lastProp.hasOwnProperty(styleName) || nextProp && nextProp.hasOwnProperty(styleName) || (styleUpdates1 || (styleUpdates1 = {}), styleUpdates1[styleName] = "");
|
||||
for(styleName in nextProp)nextProp.hasOwnProperty(styleName) && lastProp[styleName] !== nextProp[styleName] && (styleUpdates1 || (styleUpdates1 = {}), styleUpdates1[styleName] = nextProp[styleName]);
|
||||
} else styleUpdates1 || (updatePayload || (updatePayload = []), updatePayload.push(propKey, styleUpdates1)), styleUpdates1 = nextProp;
|
||||
} else if (propKey === DANGEROUSLY_SET_INNER_HTML) {
|
||||
var nextHtml = nextProp ? nextProp[HTML$1] : void 0, lastHtml = lastProp ? lastProp[HTML$1] : void 0;
|
||||
null != nextHtml && lastHtml !== nextHtml && (updatePayload = updatePayload || []).push(propKey, nextHtml);
|
||||
} else propKey === CHILDREN ? ("string" == typeof nextProp || "number" == typeof nextProp) && (updatePayload = updatePayload || []).push(propKey, "" + nextProp) : propKey !== SUPPRESS_CONTENT_EDITABLE_WARNING && propKey !== SUPPRESS_HYDRATION_WARNING && (registrationNameDependencies1.hasOwnProperty(propKey) ? (null != nextProp && ("function" != typeof nextProp && warnForInvalidEventListener(propKey, nextProp), "onScroll" === propKey && listenToNonDelegatedEvent("scroll", domElement)), updatePayload || lastProp === nextProp || (updatePayload = [])) : "object" == typeof nextProp && null !== nextProp && nextProp.$$typeof === REACT_OPAQUE_ID_TYPE ? nextProp.toString() : (updatePayload = updatePayload || []).push(propKey, nextProp));
|
||||
}
|
||||
}
|
||||
}(styleUpdates1, nextProps[STYLE]), (updatePayload = updatePayload || []).push(STYLE, styleUpdates1)), updatePayload;
|
||||
}(domElement5, type13, oldProps1, newProps3));
|
||||
return styleUpdates1 && (function(styleUpdates, nextStyles) {
|
||||
if (nextStyles) {
|
||||
var expandedUpdates = expandShorthandMap(styleUpdates), expandedStyles = expandShorthandMap(nextStyles), warnedAbout = {};
|
||||
for(var key in expandedUpdates){
|
||||
var originalKey = expandedUpdates[key], correctOriginalKey = expandedStyles[key];
|
||||
if (correctOriginalKey && originalKey !== correctOriginalKey) {
|
||||
var warningKey = originalKey + "," + correctOriginalKey;
|
||||
if (warnedAbout[warningKey]) continue;
|
||||
warnedAbout[warningKey] = !0, error1("%s a style property during rerender (%s) when a conflicting property is set (%s) can lead to styling bugs. To avoid this, don't mix shorthand and non-shorthand properties for the same value; instead, replace the shorthand with separate values.", isValueEmpty(styleUpdates[originalKey]) ? "Removing" : "Updating", originalKey, correctOriginalKey);
|
||||
}
|
||||
}
|
||||
}
|
||||
}(styleUpdates1, nextProps[STYLE]), (updatePayload = updatePayload || []).push(STYLE, styleUpdates1)), updatePayload;
|
||||
}(domElement5, type, oldProps, newProps);
|
||||
}(instance, type13, oldProps1, newProps3, rootContainerInstance, currentHostContext);
|
||||
workInProgress.updateQueue = updatePayload3, updatePayload3 && markUpdate(workInProgress);
|
||||
}
|
||||
}, updateHostText$1 = function(current, workInProgress, oldText, newText) {
|
||||
@ -7533,10 +7578,20 @@
|
||||
};
|
||||
function safelyDetachRef(current) {
|
||||
var ref = current.ref;
|
||||
null !== ref && ("function" == typeof ref ? (invokeGuardedCallback(null, ref, null, null), hasError && captureCommitPhaseError(current, clearCaughtError())) : ref.current = null);
|
||||
if (null !== ref) {
|
||||
if ("function" == typeof ref) {
|
||||
if (invokeGuardedCallback(null, ref, null, null), hasError) {
|
||||
var refError = clearCaughtError();
|
||||
captureCommitPhaseError(current, refError);
|
||||
}
|
||||
} else ref.current = null;
|
||||
}
|
||||
}
|
||||
function safelyCallDestroy(current, destroy) {
|
||||
invokeGuardedCallback(null, destroy, null), hasError && captureCommitPhaseError(current, clearCaughtError());
|
||||
if (invokeGuardedCallback(null, destroy, null), hasError) {
|
||||
var error = clearCaughtError();
|
||||
captureCommitPhaseError(current, error);
|
||||
}
|
||||
}
|
||||
function commitBeforeMutationLifeCycles(current, finishedWork) {
|
||||
switch(finishedWork.tag){
|
||||
@ -7678,41 +7733,46 @@
|
||||
var currentRef = current.ref;
|
||||
null !== currentRef && ("function" == typeof currentRef ? currentRef(null) : currentRef.current = null);
|
||||
}
|
||||
function commitUnmount(finishedRoot, current, renderPriorityLevel) {
|
||||
function commitUnmount(finishedRoot, current14, renderPriorityLevel) {
|
||||
switch(!function(fiber) {
|
||||
if (injectedHook && "function" == typeof injectedHook.onCommitFiberUnmount) try {
|
||||
injectedHook.onCommitFiberUnmount(rendererID, fiber);
|
||||
} catch (err) {
|
||||
hasLoggedError || (hasLoggedError = !0, error1("React instrumentation encountered an error: %s", err));
|
||||
}
|
||||
}(current), current.tag){
|
||||
}(current14), current14.tag){
|
||||
case 0:
|
||||
case 11:
|
||||
case 14:
|
||||
case 15:
|
||||
case 22:
|
||||
var updateQueue = current.updateQueue;
|
||||
var updateQueue = current14.updateQueue;
|
||||
if (null !== updateQueue) {
|
||||
var lastEffect = updateQueue.lastEffect;
|
||||
if (null !== lastEffect) {
|
||||
var firstEffect = lastEffect.next, effect = firstEffect;
|
||||
do {
|
||||
var _effect2 = effect, destroy = _effect2.destroy, tag = _effect2.tag;
|
||||
void 0 !== destroy && ((4 & tag) != 0 ? enqueuePendingPassiveHookEffectUnmount(current, effect) : safelyCallDestroy(current, destroy)), effect = effect.next;
|
||||
void 0 !== destroy && ((4 & tag) != 0 ? enqueuePendingPassiveHookEffectUnmount(current14, effect) : safelyCallDestroy(current14, destroy)), effect = effect.next;
|
||||
}while (effect !== firstEffect)
|
||||
}
|
||||
}
|
||||
return;
|
||||
case 1:
|
||||
safelyDetachRef(current);
|
||||
var current14, instance, instance10 = current.stateNode;
|
||||
"function" != typeof instance10.componentWillUnmount || (current14 = current, invokeGuardedCallback(null, callComponentWillUnmountWithTimer, null, current14, instance = instance10), hasError && captureCommitPhaseError(current14, clearCaughtError()));
|
||||
safelyDetachRef(current14);
|
||||
var instance10 = current14.stateNode;
|
||||
"function" == typeof instance10.componentWillUnmount && function(current, instance) {
|
||||
if (invokeGuardedCallback(null, callComponentWillUnmountWithTimer, null, current, instance), hasError) {
|
||||
var unmountError = clearCaughtError();
|
||||
captureCommitPhaseError(current, unmountError);
|
||||
}
|
||||
}(current14, instance10);
|
||||
return;
|
||||
case 5:
|
||||
safelyDetachRef(current);
|
||||
safelyDetachRef(current14);
|
||||
return;
|
||||
case 4:
|
||||
unmountHostComponents(finishedRoot, current);
|
||||
unmountHostComponents(finishedRoot, current14);
|
||||
return;
|
||||
case 20:
|
||||
case 18:
|
||||
@ -7880,26 +7940,26 @@
|
||||
case 5:
|
||||
var instance = finishedWork2.stateNode;
|
||||
if (null != instance) {
|
||||
var domElement7, updatePayload6, type, oldProps, newProps, newProps4 = finishedWork2.memoizedProps, oldProps2 = null !== current ? current.memoizedProps : newProps4, type15 = finishedWork2.type, updatePayload5 = finishedWork2.updateQueue;
|
||||
finishedWork2.updateQueue = null, null !== updatePayload5 && (domElement7 = instance, updatePayload6 = updatePayload5, type = type15, oldProps = oldProps2, updateFiberProps(domElement7, newProps = newProps4), function(domElement9, updatePayload8, tag, lastRawProps, nextRawProps) {
|
||||
"input" === tag && "radio" === nextRawProps.type && null != nextRawProps.name && updateChecked(domElement9, nextRawProps);
|
||||
var domElement6, updatePayload6, type, oldProps, newProps, newProps4 = finishedWork2.memoizedProps, oldProps2 = null !== current ? current.memoizedProps : newProps4, type15 = finishedWork2.type, updatePayload5 = finishedWork2.updateQueue;
|
||||
finishedWork2.updateQueue = null, null !== updatePayload5 && (domElement6 = instance, updatePayload6 = updatePayload5, type = type15, oldProps = oldProps2, updateFiberProps(domElement6, newProps = newProps4), function(domElement8, updatePayload8, tag, lastRawProps, nextRawProps) {
|
||||
"input" === tag && "radio" === nextRawProps.type && null != nextRawProps.name && updateChecked(domElement8, nextRawProps);
|
||||
var element, props, node, wasMultiple, value, wasCustomComponentTag = isCustomComponent(tag, lastRawProps), isCustomComponentTag2 = isCustomComponent(tag, nextRawProps);
|
||||
switch(function(domElement, updatePayload, wasCustomComponentTag, isCustomComponentTag) {
|
||||
for(var i = 0; i < updatePayload.length; i += 2){
|
||||
var propKey = updatePayload[i], propValue = updatePayload[i + 1];
|
||||
propKey === STYLE ? setValueForStyles(domElement, propValue) : propKey === DANGEROUSLY_SET_INNER_HTML ? setInnerHTML(domElement, propValue) : propKey === CHILDREN ? setTextContent(domElement, propValue) : setValueForProperty(domElement, propKey, propValue, isCustomComponentTag);
|
||||
}
|
||||
}(domElement9, updatePayload8, wasCustomComponentTag, isCustomComponentTag2), tag){
|
||||
}(domElement8, updatePayload8, wasCustomComponentTag, isCustomComponentTag2), tag){
|
||||
case "input":
|
||||
updateWrapper(domElement9, nextRawProps);
|
||||
updateWrapper(domElement8, nextRawProps);
|
||||
break;
|
||||
case "textarea":
|
||||
updateWrapper$1(domElement9, nextRawProps);
|
||||
updateWrapper$1(domElement8, nextRawProps);
|
||||
break;
|
||||
case "select":
|
||||
element = domElement9, props = nextRawProps, wasMultiple = (node = element)._wrapperState.wasMultiple, node._wrapperState.wasMultiple = !!props.multiple, value = props.value, null != value ? updateOptions(node, !!props.multiple, value, !1) : !!props.multiple !== wasMultiple && (null != props.defaultValue ? updateOptions(node, !!props.multiple, props.defaultValue, !0) : updateOptions(node, !!props.multiple, props.multiple ? [] : "", !1));
|
||||
element = domElement8, props = nextRawProps, wasMultiple = (node = element)._wrapperState.wasMultiple, node._wrapperState.wasMultiple = !!props.multiple, value = props.value, null != value ? updateOptions(node, !!props.multiple, value, !1) : !!props.multiple !== wasMultiple && (null != props.defaultValue ? updateOptions(node, !!props.multiple, props.defaultValue, !0) : updateOptions(node, !!props.multiple, props.multiple ? [] : "", !1));
|
||||
}
|
||||
}(domElement7, updatePayload6, type, oldProps, newProps));
|
||||
}(domElement6, updatePayload6, type, oldProps, newProps));
|
||||
}
|
||||
return;
|
||||
case 6:
|
||||
@ -7985,21 +8045,26 @@
|
||||
if ((4 & mode) == 0) return 99 === getCurrentPriorityLevel() ? SyncLane : 2;
|
||||
if (currentEventWipLanes === NoLanes && (currentEventWipLanes = workInProgressRootIncludedLanes), 0 !== ReactCurrentBatchConfig.transition) return currentEventPendingLanes !== NoLanes && (currentEventPendingLanes = null !== mostRecentlyUpdatedRoot ? mostRecentlyUpdatedRoot.pendingLanes : NoLanes), wipLanes = currentEventWipLanes, (lane = pickArbitraryLane(4186112 & ~currentEventPendingLanes)) === NoLane && (lane = pickArbitraryLane(4186112 & ~wipLanes)) === NoLane && (lane = pickArbitraryLane(4186112)), lane;
|
||||
var schedulerPriority = getCurrentPriorityLevel();
|
||||
return (4 & executionContext) != 0 && 98 === schedulerPriority ? findUpdateLane(12, currentEventWipLanes) : findUpdateLane(function(schedulerPriorityLevel) {
|
||||
switch(schedulerPriorityLevel){
|
||||
case 99:
|
||||
return 15;
|
||||
case 98:
|
||||
return 10;
|
||||
case 97:
|
||||
case 96:
|
||||
return 8;
|
||||
case 95:
|
||||
return 2;
|
||||
default:
|
||||
return 0;
|
||||
}
|
||||
}(schedulerPriority), currentEventWipLanes);
|
||||
if ((4 & executionContext) != 0 && 98 === schedulerPriority) lane1 = findUpdateLane(12, currentEventWipLanes);
|
||||
else {
|
||||
var schedulerLanePriority = function(schedulerPriorityLevel) {
|
||||
switch(schedulerPriorityLevel){
|
||||
case 99:
|
||||
return 15;
|
||||
case 98:
|
||||
return 10;
|
||||
case 97:
|
||||
case 96:
|
||||
return 8;
|
||||
case 95:
|
||||
return 2;
|
||||
default:
|
||||
return 0;
|
||||
}
|
||||
}(schedulerPriority);
|
||||
lane1 = findUpdateLane(schedulerLanePriority, currentEventWipLanes);
|
||||
}
|
||||
return lane1;
|
||||
}
|
||||
function scheduleUpdateOnFiber(fiber, lane, eventTime) {
|
||||
checkForNestedUpdates(), warnAboutRenderPhaseUpdatesInDEV(fiber);
|
||||
@ -8035,35 +8100,41 @@
|
||||
if (root3.callbackPriority === newCallbackPriority) return;
|
||||
cancelCallback(existingCallbackNode);
|
||||
}
|
||||
newCallbackNode = 15 === newCallbackPriority ? (callback = performSyncWorkOnRoot.bind(null, root3), null === syncQueue ? (syncQueue = [
|
||||
if (15 === newCallbackPriority) newCallbackNode = (callback = performSyncWorkOnRoot.bind(null, root3), null === syncQueue ? (syncQueue = [
|
||||
callback
|
||||
], immediateQueueCallbackNode = Scheduler_scheduleCallback(Scheduler_ImmediatePriority, flushSyncCallbackQueueImpl)) : syncQueue.push(callback), fakeCallbackNode) : 14 === newCallbackPriority ? scheduleCallback(99, performSyncWorkOnRoot.bind(null, root3)) : scheduleCallback(function(lanePriority) {
|
||||
switch(lanePriority){
|
||||
case 15:
|
||||
case 14:
|
||||
return 99;
|
||||
case 13:
|
||||
case 12:
|
||||
case 11:
|
||||
case 10:
|
||||
return 98;
|
||||
case 9:
|
||||
case 8:
|
||||
case 7:
|
||||
case 6:
|
||||
case 4:
|
||||
case 5:
|
||||
return 97;
|
||||
case 3:
|
||||
case 2:
|
||||
case 1:
|
||||
return 95;
|
||||
case 0:
|
||||
return 90;
|
||||
default:
|
||||
throw Error("Invalid update priority: " + lanePriority + ". This is a bug in React.");
|
||||
}
|
||||
}(newCallbackPriority), performConcurrentWorkOnRoot.bind(null, root3)), root3.callbackPriority = newCallbackPriority, root3.callbackNode = newCallbackNode;
|
||||
], immediateQueueCallbackNode = Scheduler_scheduleCallback(Scheduler_ImmediatePriority, flushSyncCallbackQueueImpl)) : syncQueue.push(callback), fakeCallbackNode);
|
||||
else if (14 === newCallbackPriority) newCallbackNode = scheduleCallback(99, performSyncWorkOnRoot.bind(null, root3));
|
||||
else {
|
||||
var schedulerPriorityLevel = function(lanePriority) {
|
||||
switch(lanePriority){
|
||||
case 15:
|
||||
case 14:
|
||||
return 99;
|
||||
case 13:
|
||||
case 12:
|
||||
case 11:
|
||||
case 10:
|
||||
return 98;
|
||||
case 9:
|
||||
case 8:
|
||||
case 7:
|
||||
case 6:
|
||||
case 4:
|
||||
case 5:
|
||||
return 97;
|
||||
case 3:
|
||||
case 2:
|
||||
case 1:
|
||||
return 95;
|
||||
case 0:
|
||||
return 90;
|
||||
default:
|
||||
throw Error("Invalid update priority: " + lanePriority + ". This is a bug in React.");
|
||||
}
|
||||
}(newCallbackPriority);
|
||||
newCallbackNode = scheduleCallback(schedulerPriorityLevel, performConcurrentWorkOnRoot.bind(null, root3));
|
||||
}
|
||||
root3.callbackPriority = newCallbackPriority, root3.callbackNode = newCallbackNode;
|
||||
}
|
||||
function performConcurrentWorkOnRoot(root) {
|
||||
if (currentEventTime = -1, currentEventWipLanes = NoLanes, currentEventPendingLanes = NoLanes, (48 & executionContext) != 0) throw Error("Should not already be working.");
|
||||
@ -8385,13 +8456,15 @@
|
||||
}, setEnabled(!1), null), shouldFireAfterActiveInstanceBlur = !1, nextEffect = firstEffect;
|
||||
do if (invokeGuardedCallback(null, commitBeforeMutationEffects, null), hasError) {
|
||||
if (!(null !== nextEffect)) throw Error("Should be working on an effect.");
|
||||
captureCommitPhaseError(nextEffect, clearCaughtError()), nextEffect = nextEffect.nextEffect;
|
||||
var error = clearCaughtError();
|
||||
captureCommitPhaseError(nextEffect, error), nextEffect = nextEffect.nextEffect;
|
||||
}
|
||||
while (null !== nextEffect)
|
||||
focusedInstanceHandle = null, recordCommitTime(), nextEffect = firstEffect;
|
||||
do if (invokeGuardedCallback(null, commitMutationEffects, null, root6, renderPriorityLevel), hasError) {
|
||||
if (!(null !== nextEffect)) throw Error("Should be working on an effect.");
|
||||
captureCommitPhaseError(nextEffect, clearCaughtError()), nextEffect = nextEffect.nextEffect;
|
||||
var _error = clearCaughtError();
|
||||
captureCommitPhaseError(nextEffect, _error), nextEffect = nextEffect.nextEffect;
|
||||
}
|
||||
while (null !== nextEffect)
|
||||
root6.containerInfo, function(priorSelectionInformation) {
|
||||
@ -8427,7 +8500,8 @@
|
||||
}(selectionInformation), setEnabled(eventsEnabled), eventsEnabled = null, selectionInformation = null, root6.current = finishedWork, nextEffect = firstEffect;
|
||||
do if (invokeGuardedCallback(null, commitLayoutEffects, null, root6, lanes7), hasError) {
|
||||
if (!(null !== nextEffect)) throw Error("Should be working on an effect.");
|
||||
captureCommitPhaseError(nextEffect, clearCaughtError()), nextEffect = nextEffect.nextEffect;
|
||||
var _error2 = clearCaughtError();
|
||||
captureCommitPhaseError(nextEffect, _error2), nextEffect = nextEffect.nextEffect;
|
||||
}
|
||||
while (null !== nextEffect)
|
||||
nextEffect = null, requestPaint(), popInteractions(prevInteractions), executionContext = prevExecutionContext;
|
||||
@ -8549,7 +8623,8 @@
|
||||
if (null !== alternate && (alternate.flags &= -8193), "function" == typeof destroy) {
|
||||
if (setCurrentFiber(fiber), invokeGuardedCallback(null, destroy, null), hasError) {
|
||||
if (!(null !== fiber)) throw Error("Should be working on an effect.");
|
||||
captureCommitPhaseError(fiber, clearCaughtError());
|
||||
var error = clearCaughtError();
|
||||
captureCommitPhaseError(fiber, error);
|
||||
}
|
||||
resetCurrentFiber();
|
||||
}
|
||||
@ -8560,7 +8635,8 @@
|
||||
var _effect2 = mountEffects[_i], _fiber = mountEffects[_i + 1];
|
||||
if (setCurrentFiber(_fiber), invokeGuardedCallback(null, invokePassiveEffectCreate, null, _effect2), hasError) {
|
||||
if (!(null !== _fiber)) throw Error("Should be working on an effect.");
|
||||
captureCommitPhaseError(_fiber, clearCaughtError());
|
||||
var _error4 = clearCaughtError();
|
||||
captureCommitPhaseError(_fiber, _error4);
|
||||
}
|
||||
resetCurrentFiber();
|
||||
}
|
||||
@ -8582,7 +8658,7 @@
|
||||
hasUncaughtError || (hasUncaughtError = !0, firstUncaughtError = error);
|
||||
};
|
||||
function captureCommitPhaseErrorOnRoot(rootFiber, sourceFiber, error) {
|
||||
var update = createRootErrorUpdate(rootFiber, createCapturedValue(error, sourceFiber), SyncLane);
|
||||
var errorInfo = createCapturedValue(error, sourceFiber), update = createRootErrorUpdate(rootFiber, errorInfo, SyncLane);
|
||||
enqueueUpdate(rootFiber, update);
|
||||
var eventTime = requestEventTime(), root = markUpdateLaneFromFiberToRoot(rootFiber, SyncLane);
|
||||
null !== root && (markRootUpdated(root, SyncLane, eventTime), ensureRootIsScheduled(root, eventTime), schedulePendingInteractions(root, SyncLane));
|
||||
@ -8695,7 +8771,11 @@
|
||||
case 11:
|
||||
case 15:
|
||||
var renderingComponentName = workInProgress1 && getComponentName(workInProgress1.type) || "Unknown", dedupeKey = renderingComponentName;
|
||||
didWarnAboutUpdateInRenderForAnotherComponent.has(dedupeKey) || (didWarnAboutUpdateInRenderForAnotherComponent.add(dedupeKey), error1("Cannot update a component (`%s`) while rendering a different component (`%s`). To locate the bad setState() call inside `%s`, follow the stack trace as described in https://reactjs.org/link/setstate-in-render", getComponentName(fiber.type) || "Unknown", renderingComponentName, renderingComponentName));
|
||||
if (!didWarnAboutUpdateInRenderForAnotherComponent.has(dedupeKey)) {
|
||||
didWarnAboutUpdateInRenderForAnotherComponent.add(dedupeKey);
|
||||
var setStateComponentName = getComponentName(fiber.type) || "Unknown";
|
||||
error1("Cannot update a component (`%s`) while rendering a different component (`%s`). To locate the bad setState() call inside `%s`, follow the stack trace as described in https://reactjs.org/link/setstate-in-render", setStateComponentName, renderingComponentName, renderingComponentName);
|
||||
}
|
||||
break;
|
||||
case 1:
|
||||
didWarnAboutUpdateInRender || (error1("Cannot update during an existing state transition (such as within `render`). Render methods should be a pure function of props and state."), didWarnAboutUpdateInRender = !0);
|
||||
@ -9336,11 +9416,17 @@
|
||||
}, function(fn) {
|
||||
attemptUserBlockingHydration = fn;
|
||||
}(function(fiber) {
|
||||
13 === fiber.tag && (scheduleUpdateOnFiber(fiber, 4, requestEventTime()), markRetryLaneIfNotHydrated(fiber, 4));
|
||||
if (13 === fiber.tag) {
|
||||
var eventTime = requestEventTime();
|
||||
scheduleUpdateOnFiber(fiber, 4, eventTime), markRetryLaneIfNotHydrated(fiber, 4);
|
||||
}
|
||||
}), function(fn) {
|
||||
attemptContinuousHydration = fn;
|
||||
}(function(fiber) {
|
||||
13 === fiber.tag && (scheduleUpdateOnFiber(fiber, 67108864, requestEventTime()), markRetryLaneIfNotHydrated(fiber, 67108864));
|
||||
if (13 === fiber.tag) {
|
||||
var eventTime = requestEventTime();
|
||||
scheduleUpdateOnFiber(fiber, 67108864, eventTime), markRetryLaneIfNotHydrated(fiber, 67108864);
|
||||
}
|
||||
}), function(fn) {
|
||||
attemptHydrationAtCurrentPriority = fn;
|
||||
}(function(fiber) {
|
||||
|
@ -147,7 +147,8 @@
|
||||
return function(obj, value2, context) {
|
||||
var result = {}, iterator = null == value2 ? _.identity : lookupIterator(value2);
|
||||
return each(obj, function(value, index) {
|
||||
behavior(result, iterator.call(context, value, index, obj), value);
|
||||
var key = iterator.call(context, value, index, obj);
|
||||
behavior(result, key, value);
|
||||
}), result;
|
||||
};
|
||||
};
|
||||
|
@ -53,7 +53,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: true,
|
||||
@ -169,12 +169,12 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 1,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: false,
|
||||
reassigned_with_var_decl: false,
|
||||
mutated: false,
|
||||
mutated: true,
|
||||
has_property_access: false,
|
||||
has_property_mutation: false,
|
||||
accessed_props: {},
|
||||
|
@ -53,7 +53,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: true,
|
||||
@ -169,12 +169,12 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 1,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: false,
|
||||
reassigned_with_var_decl: false,
|
||||
mutated: false,
|
||||
mutated: true,
|
||||
has_property_access: false,
|
||||
has_property_mutation: false,
|
||||
accessed_props: {},
|
||||
|
@ -91,7 +91,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 1,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: true,
|
||||
|
@ -13,12 +13,12 @@ TestSnapshot {
|
||||
declared_count: 0,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 0,
|
||||
assign_count: 1,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 3,
|
||||
reassigned_with_assignment: false,
|
||||
reassigned_with_var_decl: false,
|
||||
mutated: false,
|
||||
mutated: true,
|
||||
has_property_access: true,
|
||||
has_property_mutation: false,
|
||||
accessed_props: {},
|
||||
@ -127,7 +127,7 @@ TestSnapshot {
|
||||
declared_count: 1,
|
||||
declared_as_fn_param: false,
|
||||
declared_as_fn_expr: false,
|
||||
assign_count: 1,
|
||||
assign_count: 2,
|
||||
mutation_by_call_count: 0,
|
||||
usage_count: 2,
|
||||
reassigned_with_assignment: true,
|
||||
|
@ -34,21 +34,12 @@ use testing::assert_eq;
|
||||
#[testing::fixture(
|
||||
"tests/terser/compress/**/input.js",
|
||||
exclude(
|
||||
"collapse_vars/issue_1631_1/",
|
||||
"collapse_vars/issue_1631_2/",
|
||||
"collapse_vars/issue_1631_3/",
|
||||
"dead_code/try_catch_finally/",
|
||||
"drop_unused/issue_1715_1/",
|
||||
"drop_unused/issue_1715_2/",
|
||||
"drop_unused/issue_1715_3/",
|
||||
"evaluate/issue_1760_1/",
|
||||
"functions/issue_2620_4/",
|
||||
"issue_1105/assorted_Infinity_NaN_undefined_in_with_scope/",
|
||||
"issue_1105/assorted_Infinity_NaN_undefined_in_with_scope_keep_infinity/",
|
||||
"issue_1733/function_catch_catch/",
|
||||
"issue_1750/case_1/",
|
||||
"properties/issue_3188_3/",
|
||||
"rename/function_catch_catch/",
|
||||
"yield/issue_2689/",
|
||||
// We don't care about ie8
|
||||
"ie8",
|
||||
|
Loading…
Reference in New Issue
Block a user